From 578a0a6240aa27c6fd51e0e22ddc523c615ea062 Mon Sep 17 00:00:00 2001 From: Sebastian Ullrich Date: Wed, 24 Dec 2025 09:17:55 +0000 Subject: [PATCH 1/5] chore: introduce `@[allow_native_decide]` attribute --- src/Lean.lean | 1 + src/Lean/AllowNativeDecide.lean | 16 ++++++++++++++++ 2 files changed, 17 insertions(+) create mode 100644 src/Lean/AllowNativeDecide.lean diff --git a/src/Lean.lean b/src/Lean.lean index c708d08fb755..6f698c25c3b1 100644 --- a/src/Lean.lean +++ b/src/Lean.lean @@ -48,3 +48,4 @@ public import Lean.ErrorExplanations public import Lean.DefEqAttrib public import Lean.Shell public import Lean.ExtraModUses +public import Lean.AllowNativeDecide diff --git a/src/Lean/AllowNativeDecide.lean b/src/Lean/AllowNativeDecide.lean new file mode 100644 index 000000000000..d09133b1314b --- /dev/null +++ b/src/Lean/AllowNativeDecide.lean @@ -0,0 +1,16 @@ +/- +Copyright (c) 2025 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. +Authors: Sebastian Ullrich +-/ +module + +prelude + +public import Lean.Attributes + +namespace Lean + +builtin_initialize allowNativeDecideAttr : TagAttribute ← + registerTagAttribute `allow_native_decide + "mark definition as allowed to be used in `native_decide` computations" From 2b1fe3c3546e0d50205ba6472ce6910018af0a66 Mon Sep 17 00:00:00 2001 From: Sebastian Ullrich Date: Wed, 24 Dec 2025 11:56:20 +0000 Subject: [PATCH 2/5] chore: update stage0 --- stage0/stdlib/Init/Grind/Ordered/Linarith.c | 16 +- stage0/stdlib/Init/Grind/Ring/CommSolver.c | 22 +- stage0/stdlib/Init/System/IO.c | 56 +- stage0/stdlib/Lake/Build/Data.c | 1100 +-- stage0/stdlib/Lake/Config/Pattern.c | 28 +- stage0/stdlib/Lake/DSL/Targets.c | 7274 ++++++++--------- stage0/stdlib/Lake/Util/Url.c | 114 +- stage0/stdlib/Lake/Util/Version.c | 216 +- stage0/stdlib/Lean.c | 6 +- stage0/stdlib/Lean/AllowNativeDecide.c | 154 + stage0/stdlib/Lean/Compiler/LCNF/Basic.c | 24 +- stage0/stdlib/Lean/Compiler/LCNF/Specialize.c | 1304 +-- stage0/stdlib/Lean/Data/Json/Basic.c | 56 +- stage0/stdlib/Lean/DocString/Add.c | 250 +- stage0/stdlib/Lean/DocString/Types.c | 18 +- stage0/stdlib/Lean/Elab/Do/Legacy.c | 450 +- stage0/stdlib/Lean/Elab/DocString.c | 116 +- stage0/stdlib/Lean/Elab/DocString/Builtin.c | 886 +- stage0/stdlib/Lean/Elab/MutualInductive.c | 880 +- .../Lean/Elab/PreDefinition/MkInhabitant.c | 12 +- .../PreDefinition/Structural/FindRecArg.c | 110 +- stage0/stdlib/Lean/Elab/Structure.c | 2068 ++--- .../Elab/Tactic/Do/VCGen/SuggestInvariant.c | 18 +- stage0/stdlib/Lean/Elab/Tactic/RCases.c | 312 +- stage0/stdlib/Lean/Elab/Tactic/Try.c | 1128 +-- stage0/stdlib/Lean/Elab/Term/TermElabM.c | 1020 +-- stage0/stdlib/Lean/Level.c | 14 +- stage0/stdlib/Lean/Meta/ArgsPacker.c | 10 +- stage0/stdlib/Lean/Meta/IndPredBelow.c | 608 +- stage0/stdlib/Lean/Meta/Injective.c | 192 +- stage0/stdlib/Lean/Meta/LazyDiscrTree.c | 354 +- stage0/stdlib/Lean/Meta/Tactic/AC/Main.c | 38 +- stage0/stdlib/Lean/Meta/Tactic/Apply.c | 112 +- stage0/stdlib/Lean/Meta/Tactic/Backtrack.c | 242 +- stage0/stdlib/Lean/Meta/Tactic/FunInd.c | 2248 ++--- stage0/stdlib/Lean/Meta/Tactic/Grind/AC/Eq.c | 230 +- stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c | 1872 ++--- .../stdlib/Lean/Meta/Tactic/Grind/MatchCond.c | 616 +- .../Completion/CompletionItemCompression.c | 124 +- stage0/stdlib/Lean/Server/FileWorker.c | 788 +- stage0/stdlib/Lean/Server/Test/Runner.c | 820 +- stage0/stdlib/Lean/Server/Watchdog.c | 306 +- .../Lean/Widget/InteractiveDiagnostic.c | 1004 +-- .../Std/Data/DTreeMap/Internal/Balancing.c | 144 +- .../Std/Data/DTreeMap/Internal/Operations.c | 674 +- .../Bitblast/BVExpr/Circuit/Impl/Expr.c | 104 +- .../BVExpr/Circuit/Impl/Operations/Mul.c | 20 +- stage0/stdlib/Std/Time/Format/Basic.c | 492 +- 48 files changed, 13845 insertions(+), 14805 deletions(-) create mode 100644 stage0/stdlib/Lean/AllowNativeDecide.c diff --git a/stage0/stdlib/Init/Grind/Ordered/Linarith.c b/stage0/stdlib/Init/Grind/Ordered/Linarith.c index 7a1039eec930..a36db61d8fe8 100644 --- a/stage0/stdlib/Init/Grind/Ordered/Linarith.c +++ b/stage0/stdlib/Init/Grind/Ordered/Linarith.c @@ -1885,10 +1885,10 @@ lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean x_22 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_22, 0, x_18); lean_ctor_set(x_22, 1, x_21); -lean_inc(x_19); +lean_inc(x_20); x_23 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); +lean_ctor_set(x_23, 1, x_20); x_24 = l_Nat_reprFast(x_15); x_25 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_25, 0, x_24); @@ -1897,13 +1897,13 @@ lean_ctor_set(x_26, 0, x_23); lean_ctor_set(x_26, 1, x_25); x_27 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_19); +lean_ctor_set(x_27, 1, x_20); x_28 = l_Lean_Grind_Linarith_instReprPoly_repr(x_16, x_17); x_29 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); x_30 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_30, 0, x_20); +lean_ctor_set(x_30, 0, x_19); lean_ctor_set(x_30, 1, x_29); x_31 = 0; x_32 = lean_alloc_ctor(6, 1, 1); @@ -1927,8 +1927,8 @@ lean_dec(x_14); x_41 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_41, 0, x_40); x_18 = x_37; -x_19 = x_36; -x_20 = x_35; +x_19 = x_35; +x_20 = x_36; x_21 = x_41; goto block_34; } @@ -1941,8 +1941,8 @@ x_43 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_43, 0, x_42); x_44 = l_Repr_addAppParen(x_43, x_17); x_18 = x_37; -x_19 = x_36; -x_20 = x_35; +x_19 = x_35; +x_20 = x_36; x_21 = x_44; goto block_34; } diff --git a/stage0/stdlib/Init/Grind/Ring/CommSolver.c b/stage0/stdlib/Init/Grind/Ring/CommSolver.c index 2595aa0ca9f3..6f5ea774143a 100644 --- a/stage0/stdlib/Init/Grind/Ring/CommSolver.c +++ b/stage0/stdlib/Init/Grind/Ring/CommSolver.c @@ -5498,25 +5498,25 @@ goto block_59; { lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; x_37 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_37, 0, x_33); +lean_ctor_set(x_37, 0, x_34); lean_ctor_set(x_37, 1, x_36); -lean_inc(x_34); +lean_inc(x_35); x_38 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_34); +lean_ctor_set(x_38, 1, x_35); x_39 = l_Lean_Grind_CommRing_instReprMon_repr(x_30, x_32); x_40 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_39); x_41 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 1, x_35); x_42 = l_Lean_Grind_CommRing_instReprPoly_repr(x_31, x_32); x_43 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); x_44 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_44, 0, x_35); +lean_ctor_set(x_44, 0, x_33); lean_ctor_set(x_44, 1, x_43); x_45 = 0; x_46 = lean_alloc_ctor(6, 1, 1); @@ -5539,9 +5539,9 @@ x_54 = l_Int_repr(x_29); lean_dec(x_29); x_55 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_55, 0, x_54); -x_33 = x_51; -x_34 = x_50; -x_35 = x_49; +x_33 = x_49; +x_34 = x_51; +x_35 = x_50; x_36 = x_55; goto block_48; } @@ -5553,9 +5553,9 @@ lean_dec(x_29); x_57 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_57, 0, x_56); x_58 = l_Repr_addAppParen(x_57, x_32); -x_33 = x_51; -x_34 = x_50; -x_35 = x_49; +x_33 = x_49; +x_34 = x_51; +x_35 = x_50; x_36 = x_58; goto block_48; } diff --git a/stage0/stdlib/Init/System/IO.c b/stage0/stdlib/Init/System/IO.c index 3e4798e98303..45bf1716e59b 100644 --- a/stage0/stdlib/Init/System/IO.c +++ b/stage0/stdlib/Init/System/IO.c @@ -6213,17 +6213,17 @@ else { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_17 = lean_string_utf8_byte_size(x_12); -lean_inc(x_13); +lean_inc(x_11); lean_inc_ref(x_12); x_18 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_18, 0, x_12); -lean_ctor_set(x_18, 1, x_13); +lean_ctor_set(x_18, 1, x_11); lean_ctor_set(x_18, 2, x_17); -x_19 = l_String_Slice_Pos_prevn(x_18, x_17, x_11); +x_19 = l_String_Slice_Pos_prevn(x_18, x_17, x_13); lean_dec_ref(x_18); -x_20 = lean_string_utf8_extract(x_12, x_13, x_19); +x_20 = lean_string_utf8_extract(x_12, x_11, x_19); lean_dec(x_19); -lean_dec(x_13); +lean_dec(x_11); lean_dec_ref(x_12); x_7 = x_20; goto block_10; @@ -6275,9 +6275,9 @@ if (lean_obj_tag(x_35) == 0) uint32_t x_36; lean_dec_ref(x_34); x_36 = 65; -x_11 = x_27; +x_11 = x_28; x_12 = x_32; -x_13 = x_28; +x_13 = x_27; x_14 = x_36; goto block_21; } @@ -6294,9 +6294,9 @@ if (lean_obj_tag(x_38) == 0) { uint32_t x_39; x_39 = 65; -x_11 = x_27; +x_11 = x_28; x_12 = x_32; -x_13 = x_28; +x_13 = x_27; x_14 = x_39; goto block_21; } @@ -6308,9 +6308,9 @@ lean_inc(x_40); lean_dec_ref(x_38); x_41 = lean_unbox_uint32(x_40); lean_dec(x_40); -x_11 = x_27; +x_11 = x_28; x_12 = x_32; -x_13 = x_28; +x_13 = x_27; x_14 = x_41; goto block_21; } @@ -11099,8 +11099,8 @@ goto block_19; block_7: { uint32_t x_5; uint32_t x_6; -x_5 = lean_uint32_lor(x_3, x_4); -x_6 = lean_uint32_lor(x_2, x_5); +x_5 = lean_uint32_lor(x_2, x_4); +x_6 = lean_uint32_lor(x_3, x_5); return x_6; } block_15: @@ -11109,8 +11109,8 @@ if (x_10 == 0) { uint32_t x_13; x_13 = 0; -x_2 = x_11; -x_3 = x_12; +x_2 = x_12; +x_3 = x_11; x_4 = x_13; goto block_7; } @@ -11118,8 +11118,8 @@ else { uint32_t x_14; x_14 = 1; -x_2 = x_11; -x_3 = x_12; +x_2 = x_12; +x_3 = x_11; x_4 = x_14; goto block_7; } @@ -12130,17 +12130,17 @@ else { lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_18 = lean_string_utf8_byte_size(x_13); -lean_inc(x_14); +lean_inc(x_12); lean_inc_ref(x_13); x_19 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_19, 0, x_13); -lean_ctor_set(x_19, 1, x_14); +lean_ctor_set(x_19, 1, x_12); lean_ctor_set(x_19, 2, x_18); -x_20 = l_String_Slice_Pos_prevn(x_19, x_18, x_12); +x_20 = l_String_Slice_Pos_prevn(x_19, x_18, x_14); lean_dec_ref(x_19); -x_21 = lean_string_utf8_extract(x_13, x_14, x_20); +x_21 = lean_string_utf8_extract(x_13, x_12, x_20); lean_dec(x_20); -lean_dec(x_14); +lean_dec(x_12); lean_dec_ref(x_13); x_8 = x_21; goto block_11; @@ -12193,9 +12193,9 @@ if (lean_obj_tag(x_36) == 0) uint32_t x_37; lean_dec_ref(x_35); x_37 = 65; -x_12 = x_28; +x_12 = x_29; x_13 = x_33; -x_14 = x_29; +x_14 = x_28; x_15 = x_37; goto block_22; } @@ -12212,9 +12212,9 @@ if (lean_obj_tag(x_39) == 0) { uint32_t x_40; x_40 = 65; -x_12 = x_28; +x_12 = x_29; x_13 = x_33; -x_14 = x_29; +x_14 = x_28; x_15 = x_40; goto block_22; } @@ -12226,9 +12226,9 @@ lean_inc(x_41); lean_dec_ref(x_39); x_42 = lean_unbox_uint32(x_41); lean_dec(x_41); -x_12 = x_28; +x_12 = x_29; x_13 = x_33; -x_14 = x_29; +x_14 = x_28; x_15 = x_42; goto block_22; } diff --git a/stage0/stdlib/Lake/Build/Data.c b/stage0/stdlib/Lake/Build/Data.c index 10c8bdfb3c85..c3646fac84f6 100644 --- a/stage0/stdlib/Lake/Build/Data.c +++ b/stage0/stdlib/Lake/Build/Data.c @@ -1479,188 +1479,188 @@ goto block_120; block_103: { 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_inc_ref(x_20); -x_23 = l_Array_append___redArg(x_20, x_22); +lean_inc_ref(x_15); +x_23 = l_Array_append___redArg(x_15, x_22); lean_dec_ref(x_22); -lean_inc(x_18); -lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_19); x_24 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_24, 0, x_15); -lean_ctor_set(x_24, 1, x_18); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_14); lean_ctor_set(x_24, 2, x_23); x_25 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__0; -lean_inc(x_15); +lean_inc(x_19); x_26 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_26, 0, x_15); +lean_ctor_set(x_26, 0, x_19); lean_ctor_set(x_26, 1, x_25); x_27 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_15); +lean_inc(x_19); x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_15); +lean_ctor_set(x_28, 0, x_19); lean_ctor_set(x_28, 1, x_27); x_29 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__2; -lean_inc(x_15); +lean_inc(x_19); x_30 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_30, 0, x_15); +lean_ctor_set(x_30, 0, x_19); lean_ctor_set(x_30, 1, x_29); lean_inc(x_13); lean_inc_ref(x_30); -lean_inc(x_17); +lean_inc(x_16); lean_inc_ref(x_28); -lean_inc(x_15); -x_31 = l_Lean_Syntax_node8(x_15, x_19, x_24, x_26, x_11, x_28, x_14, x_17, x_30, x_13); +lean_inc(x_19); +x_31 = l_Lean_Syntax_node8(x_19, x_18, x_24, x_26, x_11, x_28, x_20, x_16, x_30, x_13); x_32 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__7; x_33 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__9; -lean_inc(x_18); -lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_19); x_34 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_34, 0, x_15); -lean_ctor_set(x_34, 1, x_18); -lean_ctor_set(x_34, 2, x_20); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_14); +lean_ctor_set(x_34, 2, x_15); x_35 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__10; x_36 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__11; -lean_inc(x_15); +lean_inc(x_19); x_37 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_37, 0, x_15); +lean_ctor_set(x_37, 0, x_19); lean_ctor_set(x_37, 1, x_35); -lean_inc(x_15); -x_38 = l_Lean_Syntax_node1(x_15, x_36, x_37); -lean_inc(x_18); -lean_inc(x_15); -x_39 = l_Lean_Syntax_node1(x_15, x_18, x_38); +lean_inc(x_19); +x_38 = l_Lean_Syntax_node1(x_19, x_36, x_37); +lean_inc(x_14); +lean_inc(x_19); +x_39 = l_Lean_Syntax_node1(x_19, x_14, x_38); lean_inc_ref_n(x_34, 6); -lean_inc(x_15); -x_40 = l_Lean_Syntax_node7(x_15, x_33, x_34, x_34, x_39, x_34, x_34, x_34, x_34); +lean_inc(x_19); +x_40 = l_Lean_Syntax_node7(x_19, x_33, x_34, x_34, x_39, x_34, x_34, x_34, x_34); x_41 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__12; x_42 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__13; x_43 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__16; lean_inc_ref(x_34); -lean_inc(x_15); -x_44 = l_Lean_Syntax_node1(x_15, x_43, x_34); -lean_inc(x_15); +lean_inc(x_19); +x_44 = l_Lean_Syntax_node1(x_19, x_43, x_34); +lean_inc(x_19); x_45 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_45, 0, x_15); +lean_ctor_set(x_45, 0, x_19); lean_ctor_set(x_45, 1, x_41); x_46 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__18; x_47 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__20; x_48 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__22; x_49 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__24; x_50 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__25; +lean_inc(x_17); lean_inc(x_21); -lean_inc(x_16); -x_51 = l_Lean_addMacroScope(x_16, x_50, x_21); +x_51 = l_Lean_addMacroScope(x_21, x_50, x_17); x_52 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__30; -lean_inc(x_15); +lean_inc(x_19); x_53 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_53, 0, x_15); +lean_ctor_set(x_53, 0, x_19); lean_ctor_set(x_53, 1, x_49); lean_ctor_set(x_53, 2, x_51); lean_ctor_set(x_53, 3, x_52); -lean_inc(x_18); -lean_inc(x_15); -x_54 = l_Lean_Syntax_node1(x_15, x_18, x_13); -lean_inc(x_15); -x_55 = l_Lean_Syntax_node2(x_15, x_48, x_53, x_54); -lean_inc(x_15); -x_56 = l_Lean_Syntax_node2(x_15, x_47, x_28, x_55); +lean_inc(x_14); +lean_inc(x_19); +x_54 = l_Lean_Syntax_node1(x_19, x_14, x_13); +lean_inc(x_19); +x_55 = l_Lean_Syntax_node2(x_19, x_48, x_53, x_54); +lean_inc(x_19); +x_56 = l_Lean_Syntax_node2(x_19, x_47, x_28, x_55); lean_inc_ref(x_34); -lean_inc(x_15); -x_57 = l_Lean_Syntax_node2(x_15, x_46, x_34, x_56); +lean_inc(x_19); +x_57 = l_Lean_Syntax_node2(x_19, x_46, x_34, x_56); x_58 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__32; x_59 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__34; x_60 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__35; -lean_inc(x_15); +lean_inc(x_19); x_61 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_61, 0, x_15); +lean_ctor_set(x_61, 0, x_19); lean_ctor_set(x_61, 1, x_60); x_62 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__36; -lean_inc(x_15); +lean_inc(x_19); x_63 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_63, 0, x_15); +lean_ctor_set(x_63, 0, x_19); lean_ctor_set(x_63, 1, x_62); x_64 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__38; x_65 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__39; -lean_inc(x_15); +lean_inc(x_19); x_66 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_66, 0, x_15); +lean_ctor_set(x_66, 0, x_19); lean_ctor_set(x_66, 1, x_65); x_67 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__42; x_68 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__44; x_69 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__45; x_70 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__46; -lean_inc(x_15); +lean_inc(x_19); x_71 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_71, 0, x_15); +lean_ctor_set(x_71, 0, x_19); lean_ctor_set(x_71, 1, x_69); x_72 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__48; lean_inc_ref(x_34); -lean_inc(x_15); -x_73 = l_Lean_Syntax_node1(x_15, x_72, x_34); +lean_inc(x_19); +x_73 = l_Lean_Syntax_node1(x_19, x_72, x_34); x_74 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__49; -lean_inc(x_15); +lean_inc(x_19); x_75 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_75, 0, x_15); +lean_ctor_set(x_75, 0, x_19); lean_ctor_set(x_75, 1, x_74); x_76 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__51; x_77 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__53; x_78 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__56; -x_79 = l_Lean_addMacroScope(x_16, x_78, x_21); +x_79 = l_Lean_addMacroScope(x_21, x_78, x_17); x_80 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__59; -lean_inc(x_15); +lean_inc(x_19); x_81 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_81, 0, x_15); +lean_ctor_set(x_81, 0, x_19); lean_ctor_set(x_81, 1, x_77); lean_ctor_set(x_81, 2, x_79); lean_ctor_set(x_81, 3, x_80); lean_inc_ref_n(x_34, 2); -lean_inc(x_15); -x_82 = l_Lean_Syntax_node3(x_15, x_76, x_34, x_34, x_81); -lean_inc(x_18); -lean_inc(x_15); -x_83 = l_Lean_Syntax_node1(x_15, x_18, x_82); +lean_inc(x_19); +x_82 = l_Lean_Syntax_node3(x_19, x_76, x_34, x_34, x_81); +lean_inc(x_14); +lean_inc(x_19); +x_83 = l_Lean_Syntax_node1(x_19, x_14, x_82); x_84 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__60; -lean_inc(x_15); +lean_inc(x_19); x_85 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_85, 0, x_15); +lean_ctor_set(x_85, 0, x_19); lean_ctor_set(x_85, 1, x_84); -lean_inc(x_18); -lean_inc(x_15); -x_86 = l_Lean_Syntax_node3(x_15, x_18, x_75, x_83, x_85); +lean_inc(x_14); +lean_inc(x_19); +x_86 = l_Lean_Syntax_node3(x_19, x_14, x_75, x_83, x_85); lean_inc_ref_n(x_34, 3); -lean_inc(x_15); -x_87 = l_Lean_Syntax_node6(x_15, x_70, x_71, x_73, x_34, x_34, x_86, x_34); -lean_inc(x_18); -lean_inc(x_15); -x_88 = l_Lean_Syntax_node1(x_15, x_18, x_87); -lean_inc(x_15); -x_89 = l_Lean_Syntax_node1(x_15, x_68, x_88); -lean_inc(x_15); -x_90 = l_Lean_Syntax_node1(x_15, x_67, x_89); -lean_inc(x_15); -x_91 = l_Lean_Syntax_node2(x_15, x_64, x_66, x_90); -lean_inc(x_18); -lean_inc(x_15); -x_92 = l_Lean_Syntax_node3(x_15, x_18, x_17, x_63, x_91); +lean_inc(x_19); +x_87 = l_Lean_Syntax_node6(x_19, x_70, x_71, x_73, x_34, x_34, x_86, x_34); +lean_inc(x_14); +lean_inc(x_19); +x_88 = l_Lean_Syntax_node1(x_19, x_14, x_87); +lean_inc(x_19); +x_89 = l_Lean_Syntax_node1(x_19, x_68, x_88); +lean_inc(x_19); +x_90 = l_Lean_Syntax_node1(x_19, x_67, x_89); +lean_inc(x_19); +x_91 = l_Lean_Syntax_node2(x_19, x_64, x_66, x_90); +lean_inc(x_14); +lean_inc(x_19); +x_92 = l_Lean_Syntax_node3(x_19, x_14, x_16, x_63, x_91); x_93 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__61; -lean_inc(x_15); +lean_inc(x_19); x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_15); +lean_ctor_set(x_94, 0, x_19); lean_ctor_set(x_94, 1, x_93); -lean_inc(x_15); -x_95 = l_Lean_Syntax_node3(x_15, x_59, x_61, x_92, x_94); +lean_inc(x_19); +x_95 = l_Lean_Syntax_node3(x_19, x_59, x_61, x_92, x_94); x_96 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__64; lean_inc_ref_n(x_34, 2); -lean_inc(x_15); -x_97 = l_Lean_Syntax_node2(x_15, x_96, x_34, x_34); +lean_inc(x_19); +x_97 = l_Lean_Syntax_node2(x_19, x_96, x_34, x_34); lean_inc_ref(x_34); -lean_inc(x_15); -x_98 = l_Lean_Syntax_node4(x_15, x_58, x_30, x_95, x_97, x_34); +lean_inc(x_19); +x_98 = l_Lean_Syntax_node4(x_19, x_58, x_30, x_95, x_97, x_34); lean_inc_ref(x_34); -lean_inc(x_15); -x_99 = l_Lean_Syntax_node6(x_15, x_42, x_44, x_45, x_34, x_34, x_57, x_98); -lean_inc(x_15); -x_100 = l_Lean_Syntax_node2(x_15, x_32, x_40, x_99); -x_101 = l_Lean_Syntax_node2(x_15, x_18, x_31, x_100); +lean_inc(x_19); +x_99 = l_Lean_Syntax_node6(x_19, x_42, x_44, x_45, x_34, x_34, x_57, x_98); +lean_inc(x_19); +x_100 = l_Lean_Syntax_node2(x_19, x_32, x_40, x_99); +x_101 = l_Lean_Syntax_node2(x_19, x_14, x_31, x_100); x_102 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_102, 0, x_101); lean_ctor_set(x_102, 1, x_3); @@ -1694,14 +1694,14 @@ x_117 = lean_ctor_get(x_104, 0); lean_inc(x_117); lean_dec_ref(x_104); x_118 = l_Array_mkArray1___redArg(x_117); -x_14 = x_110; -x_15 = x_113; -x_16 = x_105; -x_17 = x_112; -x_18 = x_114; -x_19 = x_115; -x_20 = x_116; -x_21 = x_106; +x_14 = x_114; +x_15 = x_116; +x_16 = x_112; +x_17 = x_106; +x_18 = x_115; +x_19 = x_113; +x_20 = x_110; +x_21 = x_105; x_22 = x_118; goto block_103; } @@ -1710,14 +1710,14 @@ else lean_object* x_119; lean_dec(x_104); x_119 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_14 = x_110; -x_15 = x_113; -x_16 = x_105; -x_17 = x_112; -x_18 = x_114; -x_19 = x_115; -x_20 = x_116; -x_21 = x_106; +x_14 = x_114; +x_15 = x_116; +x_16 = x_112; +x_17 = x_106; +x_18 = x_115; +x_19 = x_113; +x_20 = x_110; +x_21 = x_105; x_22 = x_119; goto block_103; } @@ -2468,239 +2468,239 @@ goto block_234; block_184: { 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_inc_ref(x_32); -x_37 = l_Array_append___redArg(x_32, x_36); +lean_inc_ref(x_30); +x_37 = l_Array_append___redArg(x_30, x_36); lean_dec_ref(x_36); -lean_inc(x_27); -lean_inc(x_34); +lean_inc(x_25); +lean_inc(x_21); x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_34); -lean_ctor_set(x_38, 1, x_27); +lean_ctor_set(x_38, 0, x_21); +lean_ctor_set(x_38, 1, x_25); lean_ctor_set(x_38, 2, x_37); x_39 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__14; x_40 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__0; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_41 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_40); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_41 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_40); x_42 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__1; -lean_inc(x_34); +lean_inc(x_21); x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_34); +lean_ctor_set(x_43, 0, x_21); lean_ctor_set(x_43, 1, x_42); x_44 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__2; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_45 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_44); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_45 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_44); x_46 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__15; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_47 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_46); -lean_inc(x_27); -lean_inc(x_34); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_47 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_46); +lean_inc(x_25); +lean_inc(x_21); x_48 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_48, 0, x_34); -lean_ctor_set(x_48, 1, x_27); -lean_ctor_set(x_48, 2, x_32); +lean_ctor_set(x_48, 0, x_21); +lean_ctor_set(x_48, 1, x_25); +lean_ctor_set(x_48, 2, x_30); lean_inc_ref(x_48); -lean_inc(x_34); -x_49 = l_Lean_Syntax_node1(x_34, x_47, x_48); +lean_inc(x_21); +x_49 = l_Lean_Syntax_node1(x_21, x_47, x_48); x_50 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__3; x_51 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__4; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_52 = l_Lean_Name_mkStr4(x_28, x_29, x_50, x_51); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_52 = l_Lean_Name_mkStr4(x_23, x_22, x_50, x_51); x_53 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__6; x_54 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__7; -lean_inc(x_30); -lean_inc(x_21); -x_55 = l_Lean_addMacroScope(x_21, x_54, x_30); -x_56 = lean_box(0); lean_inc(x_34); +lean_inc(x_27); +x_55 = l_Lean_addMacroScope(x_27, x_54, x_34); +x_56 = lean_box(0); +lean_inc(x_21); x_57 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_57, 0, x_34); +lean_ctor_set(x_57, 0, x_21); lean_ctor_set(x_57, 1, x_53); lean_ctor_set(x_57, 2, x_55); lean_ctor_set(x_57, 3, x_56); lean_inc_ref(x_48); lean_inc(x_52); -lean_inc(x_34); -x_58 = l_Lean_Syntax_node2(x_34, x_52, x_57, x_48); +lean_inc(x_21); +x_58 = l_Lean_Syntax_node2(x_21, x_52, x_57, x_48); lean_inc(x_49); lean_inc(x_45); -lean_inc(x_34); -x_59 = l_Lean_Syntax_node2(x_34, x_45, x_49, x_58); +lean_inc(x_21); +x_59 = l_Lean_Syntax_node2(x_21, x_45, x_49, x_58); x_60 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__36; -lean_inc(x_34); +lean_inc(x_21); x_61 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_61, 0, x_34); +lean_ctor_set(x_61, 0, x_21); lean_ctor_set(x_61, 1, x_60); x_62 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__9; x_63 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__10; -lean_inc(x_30); -lean_inc(x_21); -x_64 = l_Lean_addMacroScope(x_21, x_63, x_30); lean_inc(x_34); +lean_inc(x_27); +x_64 = l_Lean_addMacroScope(x_27, x_63, x_34); +lean_inc(x_21); x_65 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_65, 0, x_34); +lean_ctor_set(x_65, 0, x_21); lean_ctor_set(x_65, 1, x_62); lean_ctor_set(x_65, 2, x_64); lean_ctor_set(x_65, 3, x_56); lean_inc_ref(x_48); -lean_inc(x_34); -x_66 = l_Lean_Syntax_node2(x_34, x_52, x_65, x_48); +lean_inc(x_21); +x_66 = l_Lean_Syntax_node2(x_21, x_52, x_65, x_48); lean_inc(x_49); -lean_inc(x_34); -x_67 = l_Lean_Syntax_node2(x_34, x_45, x_49, x_66); -lean_inc(x_27); -lean_inc(x_34); -x_68 = l_Lean_Syntax_node3(x_34, x_27, x_59, x_61, x_67); +lean_inc(x_21); +x_67 = l_Lean_Syntax_node2(x_21, x_45, x_49, x_66); +lean_inc(x_25); +lean_inc(x_21); +x_68 = l_Lean_Syntax_node3(x_21, x_25, x_59, x_61, x_67); x_69 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__60; -lean_inc(x_34); +lean_inc(x_21); x_70 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_70, 0, x_34); +lean_ctor_set(x_70, 0, x_21); lean_ctor_set(x_70, 1, x_69); -lean_inc(x_34); -x_71 = l_Lean_Syntax_node3(x_34, x_41, x_43, x_68, x_70); -lean_inc(x_27); -lean_inc(x_34); -x_72 = l_Lean_Syntax_node1(x_34, x_27, x_71); +lean_inc(x_21); +x_71 = l_Lean_Syntax_node3(x_21, x_41, x_43, x_68, x_70); +lean_inc(x_25); +lean_inc(x_21); +x_72 = l_Lean_Syntax_node1(x_21, x_25, x_71); x_73 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__10; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_74 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_73); -lean_inc(x_34); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_74 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_73); +lean_inc(x_21); x_75 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_75, 0, x_34); +lean_ctor_set(x_75, 0, x_21); lean_ctor_set(x_75, 1, x_73); -lean_inc(x_34); -x_76 = l_Lean_Syntax_node1(x_34, x_74, x_75); -lean_inc(x_27); -lean_inc(x_34); -x_77 = l_Lean_Syntax_node1(x_34, x_27, x_76); +lean_inc(x_21); +x_76 = l_Lean_Syntax_node1(x_21, x_74, x_75); +lean_inc(x_25); +lean_inc(x_21); +x_77 = l_Lean_Syntax_node1(x_21, x_25, x_76); lean_inc_ref_n(x_48, 4); lean_inc(x_77); -lean_inc(x_33); -lean_inc(x_34); -x_78 = l_Lean_Syntax_node7(x_34, x_33, x_38, x_72, x_77, x_48, x_48, x_48, x_48); +lean_inc(x_32); +lean_inc(x_21); +x_78 = l_Lean_Syntax_node7(x_21, x_32, x_38, x_72, x_77, x_48, x_48, x_48, x_48); x_79 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__11; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_80 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_79); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_80 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_79); x_81 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__12; -lean_inc(x_34); +lean_inc(x_21); x_82 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_82, 0, x_34); +lean_ctor_set(x_82, 0, x_21); lean_ctor_set(x_82, 1, x_81); x_83 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__13; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_84 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_83); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_84 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_83); x_85 = lean_mk_empty_array_with_capacity(x_1); x_86 = lean_box(2); -lean_inc(x_27); +lean_inc(x_25); x_87 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_27); +lean_ctor_set(x_87, 1, x_25); lean_ctor_set(x_87, 2, x_85); x_88 = lean_mk_empty_array_with_capacity(x_2); -x_89 = lean_array_push(x_88, x_20); +x_89 = lean_array_push(x_88, x_26); x_90 = lean_array_push(x_89, x_87); x_91 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_91, 0, x_86); lean_ctor_set(x_91, 1, x_84); lean_ctor_set(x_91, 2, x_90); x_92 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__14; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_93 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_92); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_93 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_92); lean_inc_ref_n(x_48, 2); -lean_inc(x_34); -x_94 = l_Lean_Syntax_node2(x_34, x_93, x_48, x_48); +lean_inc(x_21); +x_94 = l_Lean_Syntax_node2(x_21, x_93, x_48, x_48); x_95 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__31; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_96 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_95); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_96 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_95); x_97 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__2; -lean_inc(x_34); +lean_inc(x_21); x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_34); +lean_ctor_set(x_98, 0, x_21); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__62; x_100 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__63; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_101 = l_Lean_Name_mkStr4(x_28, x_29, x_99, x_100); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_101 = l_Lean_Name_mkStr4(x_23, x_22, x_99, x_100); lean_inc_ref_n(x_48, 2); -lean_inc(x_34); -x_102 = l_Lean_Syntax_node2(x_34, x_101, x_48, x_48); +lean_inc(x_21); +x_102 = l_Lean_Syntax_node2(x_21, x_101, x_48, x_48); lean_inc_ref(x_48); lean_inc(x_102); -lean_inc(x_31); +lean_inc(x_24); lean_inc_ref(x_98); lean_inc(x_96); -lean_inc(x_34); -x_103 = l_Lean_Syntax_node4(x_34, x_96, x_98, x_31, x_102, x_48); +lean_inc(x_21); +x_103 = l_Lean_Syntax_node4(x_21, x_96, x_98, x_24, x_102, x_48); lean_inc_ref(x_48); -lean_inc(x_34); -x_104 = l_Lean_Syntax_node5(x_34, x_80, x_82, x_91, x_94, x_103, x_48); -lean_inc(x_24); -lean_inc(x_34); -x_105 = l_Lean_Syntax_node2(x_34, x_24, x_78, x_104); +lean_inc(x_21); +x_104 = l_Lean_Syntax_node5(x_21, x_80, x_82, x_91, x_94, x_103, x_48); +lean_inc(x_29); +lean_inc(x_21); +x_105 = l_Lean_Syntax_node2(x_21, x_29, x_78, x_104); x_106 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__69; lean_inc_ref(x_3); x_107 = l_Lean_Name_mkStr2(x_3, x_106); x_108 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__0; -lean_inc(x_34); +lean_inc(x_21); x_109 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_109, 0, x_34); +lean_ctor_set(x_109, 0, x_21); lean_ctor_set(x_109, 1, x_108); x_110 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_34); +lean_inc(x_21); x_111 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_111, 0, x_34); +lean_ctor_set(x_111, 0, x_21); lean_ctor_set(x_111, 1, x_110); lean_inc(x_5); lean_inc_ref(x_98); -lean_inc(x_31); +lean_inc(x_24); lean_inc_ref(x_111); lean_inc_ref(x_48); -lean_inc(x_34); -x_112 = l_Lean_Syntax_node8(x_34, x_107, x_48, x_109, x_22, x_111, x_4, x_31, x_98, x_5); +lean_inc(x_21); +x_112 = l_Lean_Syntax_node8(x_21, x_107, x_48, x_109, x_33, x_111, x_4, x_24, x_98, x_5); lean_inc_ref_n(x_48, 6); -lean_inc(x_34); -x_113 = l_Lean_Syntax_node7(x_34, x_33, x_48, x_48, x_77, x_48, x_48, x_48, x_48); +lean_inc(x_21); +x_113 = l_Lean_Syntax_node7(x_21, x_32, x_48, x_48, x_77, x_48, x_48, x_48, x_48); x_114 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__12; -lean_inc_ref(x_35); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_115 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_114); -lean_inc(x_34); +lean_inc_ref(x_31); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_115 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_114); +lean_inc(x_21); x_116 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_116, 0, x_34); +lean_ctor_set(x_116, 0, x_21); lean_ctor_set(x_116, 1, x_114); x_117 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__17; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_118 = l_Lean_Name_mkStr4(x_28, x_29, x_35, x_117); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_118 = l_Lean_Name_mkStr4(x_23, x_22, x_31, x_117); x_119 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__19; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_120 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_119); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_120 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_119); x_121 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__21; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_122 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_121); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_122 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_121); x_123 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__15; x_124 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__16; x_125 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__17; -lean_inc(x_30); -lean_inc(x_21); -x_126 = l_Lean_addMacroScope(x_21, x_125, x_30); +lean_inc(x_34); +lean_inc(x_27); +x_126 = l_Lean_addMacroScope(x_27, x_125, x_34); lean_inc_ref(x_3); x_127 = l_Lean_Name_mkStr2(x_3, x_123); lean_inc(x_127); @@ -2715,52 +2715,52 @@ lean_ctor_set(x_130, 1, x_56); x_131 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_131, 0, x_128); lean_ctor_set(x_131, 1, x_130); -lean_inc(x_34); +lean_inc(x_21); x_132 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_132, 0, x_34); +lean_ctor_set(x_132, 0, x_21); lean_ctor_set(x_132, 1, x_124); lean_ctor_set(x_132, 2, x_126); lean_ctor_set(x_132, 3, x_131); lean_inc_ref(x_6); x_133 = l_String_toRawSubstring_x27(x_6); x_134 = l_Lean_Name_mkStr1(x_6); -lean_inc(x_30); -lean_inc(x_21); -x_135 = l_Lean_addMacroScope(x_21, x_134, x_30); +lean_inc(x_34); +lean_inc(x_27); +x_135 = l_Lean_addMacroScope(x_27, x_134, x_34); x_136 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_136, 0, x_7); lean_ctor_set(x_136, 1, x_56); x_137 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_137, 0, x_136); lean_ctor_set(x_137, 1, x_56); -lean_inc(x_34); +lean_inc(x_21); x_138 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_138, 0, x_34); +lean_ctor_set(x_138, 0, x_21); lean_ctor_set(x_138, 1, x_133); lean_ctor_set(x_138, 2, x_135); lean_ctor_set(x_138, 3, x_137); x_139 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__18; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_140 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_139); +lean_inc_ref(x_22); +lean_inc_ref(x_23); +x_140 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_139); x_141 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__19; -lean_inc_ref(x_28); -x_142 = l_Lean_Name_mkStr4(x_28, x_29, x_39, x_141); +lean_inc_ref(x_23); +x_142 = l_Lean_Name_mkStr4(x_23, x_22, x_39, x_141); x_143 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__20; -lean_inc(x_34); +lean_inc(x_21); x_144 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_144, 0, x_34); +lean_ctor_set(x_144, 0, x_21); lean_ctor_set(x_144, 1, x_143); x_145 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__22; x_146 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__24; x_147 = lean_box(0); -lean_inc(x_30); -lean_inc(x_21); -x_148 = l_Lean_addMacroScope(x_21, x_147, x_30); +lean_inc(x_34); +lean_inc(x_27); +x_148 = l_Lean_addMacroScope(x_27, x_147, x_34); x_149 = l_Lean_Name_mkStr1(x_3); x_150 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_150, 0, x_149); -x_151 = l_Lean_Name_mkStr1(x_28); +x_151 = l_Lean_Name_mkStr1(x_23); x_152 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_152, 0, x_151); x_153 = lean_alloc_ctor(1, 2, 0); @@ -2769,83 +2769,83 @@ lean_ctor_set(x_153, 1, x_56); x_154 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_154, 0, x_150); lean_ctor_set(x_154, 1, x_153); -lean_inc(x_34); +lean_inc(x_21); x_155 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_155, 0, x_34); +lean_ctor_set(x_155, 0, x_21); lean_ctor_set(x_155, 1, x_146); lean_ctor_set(x_155, 2, x_148); lean_ctor_set(x_155, 3, x_154); -lean_inc(x_34); -x_156 = l_Lean_Syntax_node1(x_34, x_145, x_155); -lean_inc(x_34); -x_157 = l_Lean_Syntax_node2(x_34, x_142, x_144, x_156); +lean_inc(x_21); +x_156 = l_Lean_Syntax_node1(x_21, x_145, x_155); +lean_inc(x_21); +x_157 = l_Lean_Syntax_node2(x_21, x_142, x_144, x_156); x_158 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__26; x_159 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__27; -lean_inc(x_34); +lean_inc(x_21); x_160 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_160, 0, x_34); +lean_ctor_set(x_160, 0, x_21); lean_ctor_set(x_160, 1, x_159); -lean_inc(x_34); -x_161 = l_Lean_Syntax_node3(x_34, x_158, x_25, x_160, x_23); +lean_inc(x_21); +x_161 = l_Lean_Syntax_node3(x_21, x_158, x_35, x_160, x_28); x_162 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__28; -lean_inc(x_34); +lean_inc(x_21); x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_34); +lean_ctor_set(x_163, 0, x_21); lean_ctor_set(x_163, 1, x_162); lean_inc_ref(x_163); lean_inc(x_157); lean_inc(x_140); -lean_inc(x_34); -x_164 = l_Lean_Syntax_node3(x_34, x_140, x_157, x_161, x_163); +lean_inc(x_21); +x_164 = l_Lean_Syntax_node3(x_21, x_140, x_157, x_161, x_163); lean_inc(x_5); lean_inc_ref(x_138); -lean_inc(x_27); -lean_inc(x_34); -x_165 = l_Lean_Syntax_node3(x_34, x_27, x_138, x_164, x_5); +lean_inc(x_25); +lean_inc(x_21); +x_165 = l_Lean_Syntax_node3(x_21, x_25, x_138, x_164, x_5); lean_inc_ref(x_132); lean_inc(x_122); -lean_inc(x_34); -x_166 = l_Lean_Syntax_node2(x_34, x_122, x_132, x_165); -lean_inc(x_34); -x_167 = l_Lean_Syntax_node2(x_34, x_120, x_111, x_166); +lean_inc(x_21); +x_166 = l_Lean_Syntax_node2(x_21, x_122, x_132, x_165); +lean_inc(x_21); +x_167 = l_Lean_Syntax_node2(x_21, x_120, x_111, x_166); lean_inc_ref(x_48); -lean_inc(x_34); -x_168 = l_Lean_Syntax_node2(x_34, x_118, x_48, x_167); +lean_inc(x_21); +x_168 = l_Lean_Syntax_node2(x_21, x_118, x_48, x_167); x_169 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__30; x_170 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__31; -x_171 = l_Lean_addMacroScope(x_21, x_170, x_30); +x_171 = l_Lean_addMacroScope(x_27, x_170, x_34); x_172 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__33; -lean_inc(x_34); +lean_inc(x_21); x_173 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_173, 0, x_34); +lean_ctor_set(x_173, 0, x_21); lean_ctor_set(x_173, 1, x_169); lean_ctor_set(x_173, 2, x_171); lean_ctor_set(x_173, 3, x_172); -lean_inc(x_27); -lean_inc(x_34); -x_174 = l_Lean_Syntax_node3(x_34, x_27, x_138, x_31, x_5); +lean_inc(x_25); +lean_inc(x_21); +x_174 = l_Lean_Syntax_node3(x_21, x_25, x_138, x_24, x_5); lean_inc(x_122); -lean_inc(x_34); -x_175 = l_Lean_Syntax_node2(x_34, x_122, x_132, x_174); -lean_inc(x_34); -x_176 = l_Lean_Syntax_node3(x_34, x_140, x_157, x_175, x_163); -lean_inc(x_27); -lean_inc(x_34); -x_177 = l_Lean_Syntax_node1(x_34, x_27, x_176); -lean_inc(x_34); -x_178 = l_Lean_Syntax_node2(x_34, x_122, x_173, x_177); +lean_inc(x_21); +x_175 = l_Lean_Syntax_node2(x_21, x_122, x_132, x_174); +lean_inc(x_21); +x_176 = l_Lean_Syntax_node3(x_21, x_140, x_157, x_175, x_163); +lean_inc(x_25); +lean_inc(x_21); +x_177 = l_Lean_Syntax_node1(x_21, x_25, x_176); +lean_inc(x_21); +x_178 = l_Lean_Syntax_node2(x_21, x_122, x_173, x_177); lean_inc_ref(x_48); -lean_inc(x_34); -x_179 = l_Lean_Syntax_node4(x_34, x_96, x_98, x_178, x_102, x_48); +lean_inc(x_21); +x_179 = l_Lean_Syntax_node4(x_21, x_96, x_98, x_178, x_102, x_48); lean_inc_ref(x_48); -lean_inc(x_34); -x_180 = l_Lean_Syntax_node6(x_34, x_115, x_49, x_116, x_48, x_48, x_168, x_179); -lean_inc(x_34); -x_181 = l_Lean_Syntax_node2(x_34, x_24, x_113, x_180); -x_182 = l_Lean_Syntax_node3(x_34, x_27, x_105, x_112, x_181); +lean_inc(x_21); +x_180 = l_Lean_Syntax_node6(x_21, x_115, x_49, x_116, x_48, x_48, x_168, x_179); +lean_inc(x_21); +x_181 = l_Lean_Syntax_node2(x_21, x_29, x_113, x_180); +x_182 = l_Lean_Syntax_node3(x_21, x_25, x_105, x_112, x_181); x_183 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_183, 0, x_182); -lean_ctor_set(x_183, 1, x_26); +lean_ctor_set(x_183, 1, x_20); return x_183; } block_206: @@ -2874,22 +2874,22 @@ x_203 = lean_ctor_get(x_9, 0); lean_inc(x_203); lean_dec_ref(x_9); x_204 = l_Array_mkArray1___redArg(x_203); -x_20 = x_189; -x_21 = x_192; -x_22 = x_185; -x_23 = x_187; -x_24 = x_200; -x_25 = x_188; -x_26 = x_191; -x_27 = x_196; -x_28 = x_197; -x_29 = x_198; -x_30 = x_193; -x_31 = x_186; -x_32 = x_202; -x_33 = x_201; -x_34 = x_195; -x_35 = x_199; +x_20 = x_191; +x_21 = x_195; +x_22 = x_198; +x_23 = x_197; +x_24 = x_186; +x_25 = x_196; +x_26 = x_189; +x_27 = x_192; +x_28 = x_185; +x_29 = x_200; +x_30 = x_202; +x_31 = x_199; +x_32 = x_201; +x_33 = x_187; +x_34 = x_193; +x_35 = x_188; x_36 = x_204; goto block_184; } @@ -2898,22 +2898,22 @@ else lean_object* x_205; lean_dec(x_9); x_205 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_20 = x_189; -x_21 = x_192; -x_22 = x_185; -x_23 = x_187; -x_24 = x_200; -x_25 = x_188; -x_26 = x_191; -x_27 = x_196; -x_28 = x_197; -x_29 = x_198; -x_30 = x_193; -x_31 = x_186; -x_32 = x_202; -x_33 = x_201; -x_34 = x_195; -x_35 = x_199; +x_20 = x_191; +x_21 = x_195; +x_22 = x_198; +x_23 = x_197; +x_24 = x_186; +x_25 = x_196; +x_26 = x_189; +x_27 = x_192; +x_28 = x_185; +x_29 = x_200; +x_30 = x_202; +x_31 = x_199; +x_32 = x_201; +x_33 = x_187; +x_34 = x_193; +x_35 = x_188; x_36 = x_205; goto block_184; } @@ -2934,8 +2934,8 @@ x_214 = lean_ctor_get(x_212, 1); lean_inc(x_214); lean_dec_ref(x_212); x_185 = x_207; -x_186 = x_209; -x_187 = x_208; +x_186 = x_208; +x_187 = x_209; x_188 = x_210; x_189 = x_213; x_190 = x_18; @@ -2982,9 +2982,9 @@ x_225 = l_Lean_Syntax_getId(x_224); x_226 = l_Lean_Name_append(x_16, x_225); x_227 = l_Lean_mkIdentFrom(x_224, x_226, x_13); lean_dec(x_224); -x_185 = x_221; +x_185 = x_218; x_186 = x_222; -x_187 = x_218; +x_187 = x_221; x_188 = x_219; x_189 = x_227; x_190 = x_18; @@ -3009,9 +3009,9 @@ x_231 = lean_string_append(x_229, x_230); x_232 = l_Lean_Name_str___override(x_16, x_231); x_233 = l_Lean_mkIdentFrom(x_10, x_232, x_13); lean_dec(x_10); -x_185 = x_221; +x_185 = x_218; x_186 = x_222; -x_187 = x_218; +x_187 = x_221; x_188 = x_219; x_189 = x_233; x_190 = x_18; @@ -3023,9 +3023,9 @@ else lean_dec(x_228); lean_dec_ref(x_216); lean_dec(x_16); -x_207 = x_221; -x_208 = x_218; -x_209 = x_222; +x_207 = x_218; +x_208 = x_222; +x_209 = x_221; x_210 = x_219; goto block_215; } @@ -3034,9 +3034,9 @@ else { lean_dec(x_216); lean_dec(x_16); -x_207 = x_221; -x_208 = x_218; -x_209 = x_222; +x_207 = x_218; +x_208 = x_222; +x_209 = x_221; x_210 = x_219; goto block_215; } @@ -3924,192 +3924,192 @@ goto block_135; block_111: { 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_inc_ref(x_19); -x_32 = l_Array_append___redArg(x_19, x_31); +lean_inc_ref(x_18); +x_32 = l_Array_append___redArg(x_18, x_31); lean_dec_ref(x_31); +lean_inc(x_27); lean_inc(x_30); -lean_inc(x_29); x_33 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_33, 0, x_29); -lean_ctor_set(x_33, 1, x_30); +lean_ctor_set(x_33, 0, x_30); +lean_ctor_set(x_33, 1, x_27); lean_ctor_set(x_33, 2, x_32); x_34 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__0; -lean_inc(x_29); +lean_inc(x_30); x_35 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_35, 0, x_29); +lean_ctor_set(x_35, 0, x_30); lean_ctor_set(x_35, 1, x_34); x_36 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_29); +lean_inc(x_30); x_37 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_37, 0, x_29); +lean_ctor_set(x_37, 0, x_30); lean_ctor_set(x_37, 1, x_36); x_38 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__2; -lean_inc(x_29); +lean_inc(x_30); x_39 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_39, 0, x_29); +lean_ctor_set(x_39, 0, x_30); lean_ctor_set(x_39, 1, x_38); lean_inc(x_17); lean_inc_ref(x_39); -lean_inc(x_23); -lean_inc_ref(x_37); lean_inc(x_29); -x_40 = l_Lean_Syntax_node8(x_29, x_20, x_33, x_35, x_27, x_37, x_18, x_23, x_39, x_17); +lean_inc_ref(x_37); +lean_inc(x_30); +x_40 = l_Lean_Syntax_node8(x_30, x_21, x_33, x_35, x_25, x_37, x_20, x_29, x_39, x_17); x_41 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__7; x_42 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__9; +lean_inc(x_27); lean_inc(x_30); -lean_inc(x_29); x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_29); -lean_ctor_set(x_43, 1, x_30); -lean_ctor_set(x_43, 2, x_19); +lean_ctor_set(x_43, 0, x_30); +lean_ctor_set(x_43, 1, x_27); +lean_ctor_set(x_43, 2, x_18); x_44 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__10; x_45 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__11; -lean_inc(x_29); +lean_inc(x_30); x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_29); +lean_ctor_set(x_46, 0, x_30); lean_ctor_set(x_46, 1, x_44); -lean_inc(x_29); -x_47 = l_Lean_Syntax_node1(x_29, x_45, x_46); lean_inc(x_30); -lean_inc(x_29); -x_48 = l_Lean_Syntax_node1(x_29, x_30, x_47); +x_47 = l_Lean_Syntax_node1(x_30, x_45, x_46); +lean_inc(x_27); +lean_inc(x_30); +x_48 = l_Lean_Syntax_node1(x_30, x_27, x_47); lean_inc_ref_n(x_43, 6); -lean_inc(x_29); -x_49 = l_Lean_Syntax_node7(x_29, x_42, x_43, x_43, x_48, x_43, x_43, x_43, x_43); +lean_inc(x_30); +x_49 = l_Lean_Syntax_node7(x_30, x_42, x_43, x_43, x_48, x_43, x_43, x_43, x_43); x_50 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__12; x_51 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__13; x_52 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__16; lean_inc_ref(x_43); -lean_inc(x_29); -x_53 = l_Lean_Syntax_node1(x_29, x_52, x_43); -lean_inc(x_29); +lean_inc(x_30); +x_53 = l_Lean_Syntax_node1(x_30, x_52, x_43); +lean_inc(x_30); x_54 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_54, 0, x_29); +lean_ctor_set(x_54, 0, x_30); lean_ctor_set(x_54, 1, x_50); x_55 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__18; x_56 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__20; x_57 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__22; x_58 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__16; x_59 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__17; -lean_inc(x_24); -lean_inc(x_21); -x_60 = l_Lean_addMacroScope(x_21, x_59, x_24); +lean_inc(x_28); +lean_inc(x_23); +x_60 = l_Lean_addMacroScope(x_23, x_59, x_28); x_61 = lean_box(0); x_62 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__facetDataDecl__1___closed__4; -lean_inc(x_29); +lean_inc(x_30); x_63 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_63, 0, x_29); +lean_ctor_set(x_63, 0, x_30); lean_ctor_set(x_63, 1, x_58); lean_ctor_set(x_63, 2, x_60); lean_ctor_set(x_63, 3, x_62); -lean_inc_ref(x_22); -x_64 = l_String_toRawSubstring_x27(x_22); -x_65 = l_Lean_Name_mkStr1(x_22); -lean_inc(x_24); -lean_inc(x_21); -x_66 = l_Lean_addMacroScope(x_21, x_65, x_24); +lean_inc_ref(x_24); +x_64 = l_String_toRawSubstring_x27(x_24); +x_65 = l_Lean_Name_mkStr1(x_24); +lean_inc(x_28); +lean_inc(x_23); +x_66 = l_Lean_addMacroScope(x_23, x_65, x_28); x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_25); +lean_ctor_set(x_67, 0, x_26); lean_ctor_set(x_67, 1, x_61); x_68 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_68, 0, x_67); lean_ctor_set(x_68, 1, x_61); -lean_inc(x_29); +lean_inc(x_30); x_69 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_69, 0, x_29); +lean_ctor_set(x_69, 0, x_30); lean_ctor_set(x_69, 1, x_64); lean_ctor_set(x_69, 2, x_66); lean_ctor_set(x_69, 3, x_68); x_70 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__facetDataDecl__1___closed__5; x_71 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__facetDataDecl__1___closed__6; x_72 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__20; -lean_inc(x_29); +lean_inc(x_30); x_73 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_73, 0, x_29); +lean_ctor_set(x_73, 0, x_30); lean_ctor_set(x_73, 1, x_72); x_74 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__22; x_75 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__24; x_76 = lean_box(0); -lean_inc(x_24); -lean_inc(x_21); -x_77 = l_Lean_addMacroScope(x_21, x_76, x_24); +lean_inc(x_28); +lean_inc(x_23); +x_77 = l_Lean_addMacroScope(x_23, x_76, x_28); x_78 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__facetDataDecl__1___closed__12; -lean_inc(x_29); +lean_inc(x_30); x_79 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_79, 0, x_29); +lean_ctor_set(x_79, 0, x_30); lean_ctor_set(x_79, 1, x_75); lean_ctor_set(x_79, 2, x_77); lean_ctor_set(x_79, 3, x_78); -lean_inc(x_29); -x_80 = l_Lean_Syntax_node1(x_29, x_74, x_79); -lean_inc(x_29); -x_81 = l_Lean_Syntax_node2(x_29, x_71, x_73, x_80); +lean_inc(x_30); +x_80 = l_Lean_Syntax_node1(x_30, x_74, x_79); +lean_inc(x_30); +x_81 = l_Lean_Syntax_node2(x_30, x_71, x_73, x_80); x_82 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__26; x_83 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__27; -lean_inc(x_29); +lean_inc(x_30); x_84 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_84, 0, x_29); +lean_ctor_set(x_84, 0, x_30); lean_ctor_set(x_84, 1, x_83); -lean_inc(x_29); -x_85 = l_Lean_Syntax_node3(x_29, x_82, x_28, x_84, x_26); +lean_inc(x_30); +x_85 = l_Lean_Syntax_node3(x_30, x_82, x_22, x_84, x_19); x_86 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__28; -lean_inc(x_29); +lean_inc(x_30); x_87 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_87, 0, x_29); +lean_ctor_set(x_87, 0, x_30); lean_ctor_set(x_87, 1, x_86); lean_inc_ref(x_87); lean_inc(x_81); -lean_inc(x_29); -x_88 = l_Lean_Syntax_node3(x_29, x_70, x_81, x_85, x_87); +lean_inc(x_30); +x_88 = l_Lean_Syntax_node3(x_30, x_70, x_81, x_85, x_87); lean_inc(x_17); lean_inc_ref(x_69); +lean_inc(x_27); lean_inc(x_30); -lean_inc(x_29); -x_89 = l_Lean_Syntax_node3(x_29, x_30, x_69, x_88, x_17); +x_89 = l_Lean_Syntax_node3(x_30, x_27, x_69, x_88, x_17); lean_inc_ref(x_63); -lean_inc(x_29); -x_90 = l_Lean_Syntax_node2(x_29, x_57, x_63, x_89); -lean_inc(x_29); -x_91 = l_Lean_Syntax_node2(x_29, x_56, x_37, x_90); +lean_inc(x_30); +x_90 = l_Lean_Syntax_node2(x_30, x_57, x_63, x_89); +lean_inc(x_30); +x_91 = l_Lean_Syntax_node2(x_30, x_56, x_37, x_90); lean_inc_ref(x_43); -lean_inc(x_29); -x_92 = l_Lean_Syntax_node2(x_29, x_55, x_43, x_91); +lean_inc(x_30); +x_92 = l_Lean_Syntax_node2(x_30, x_55, x_43, x_91); x_93 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__32; x_94 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__30; x_95 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__31; -x_96 = l_Lean_addMacroScope(x_21, x_95, x_24); +x_96 = l_Lean_addMacroScope(x_23, x_95, x_28); x_97 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__facetDataDecl__1___closed__14; -lean_inc(x_29); +lean_inc(x_30); x_98 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_98, 0, x_29); +lean_ctor_set(x_98, 0, x_30); lean_ctor_set(x_98, 1, x_94); lean_ctor_set(x_98, 2, x_96); lean_ctor_set(x_98, 3, x_97); +lean_inc(x_27); lean_inc(x_30); -lean_inc(x_29); -x_99 = l_Lean_Syntax_node3(x_29, x_30, x_69, x_23, x_17); -lean_inc(x_29); -x_100 = l_Lean_Syntax_node2(x_29, x_57, x_63, x_99); -lean_inc(x_29); -x_101 = l_Lean_Syntax_node3(x_29, x_70, x_81, x_100, x_87); +x_99 = l_Lean_Syntax_node3(x_30, x_27, x_69, x_29, x_17); lean_inc(x_30); -lean_inc(x_29); -x_102 = l_Lean_Syntax_node1(x_29, x_30, x_101); -lean_inc(x_29); -x_103 = l_Lean_Syntax_node2(x_29, x_57, x_98, x_102); +x_100 = l_Lean_Syntax_node2(x_30, x_57, x_63, x_99); +lean_inc(x_30); +x_101 = l_Lean_Syntax_node3(x_30, x_70, x_81, x_100, x_87); +lean_inc(x_27); +lean_inc(x_30); +x_102 = l_Lean_Syntax_node1(x_30, x_27, x_101); +lean_inc(x_30); +x_103 = l_Lean_Syntax_node2(x_30, x_57, x_98, x_102); x_104 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__64; lean_inc_ref_n(x_43, 2); -lean_inc(x_29); -x_105 = l_Lean_Syntax_node2(x_29, x_104, x_43, x_43); +lean_inc(x_30); +x_105 = l_Lean_Syntax_node2(x_30, x_104, x_43, x_43); lean_inc_ref(x_43); -lean_inc(x_29); -x_106 = l_Lean_Syntax_node4(x_29, x_93, x_39, x_103, x_105, x_43); +lean_inc(x_30); +x_106 = l_Lean_Syntax_node4(x_30, x_93, x_39, x_103, x_105, x_43); lean_inc_ref(x_43); -lean_inc(x_29); -x_107 = l_Lean_Syntax_node6(x_29, x_51, x_53, x_54, x_43, x_43, x_92, x_106); -lean_inc(x_29); -x_108 = l_Lean_Syntax_node2(x_29, x_41, x_49, x_107); -x_109 = l_Lean_Syntax_node2(x_29, x_30, x_40, x_108); +lean_inc(x_30); +x_107 = l_Lean_Syntax_node6(x_30, x_51, x_53, x_54, x_43, x_43, x_92, x_106); +lean_inc(x_30); +x_108 = l_Lean_Syntax_node2(x_30, x_41, x_49, x_107); +x_109 = l_Lean_Syntax_node2(x_30, x_27, x_40, 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_3); @@ -4155,19 +4155,19 @@ x_132 = lean_ctor_get(x_112, 0); lean_inc(x_132); lean_dec_ref(x_112); x_133 = l_Array_mkArray1___redArg(x_132); -x_18 = x_119; -x_19 = x_131; -x_20 = x_130; -x_21 = x_113; -x_22 = x_116; -x_23 = x_125; -x_24 = x_114; -x_25 = x_117; -x_26 = x_123; -x_27 = x_126; -x_28 = x_121; -x_29 = x_128; -x_30 = x_129; +x_18 = x_131; +x_19 = x_123; +x_20 = x_119; +x_21 = x_130; +x_22 = x_121; +x_23 = x_113; +x_24 = x_116; +x_25 = x_126; +x_26 = x_117; +x_27 = x_129; +x_28 = x_114; +x_29 = x_125; +x_30 = x_128; x_31 = x_133; goto block_111; } @@ -4176,19 +4176,19 @@ else lean_object* x_134; lean_dec(x_112); x_134 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_18 = x_119; -x_19 = x_131; -x_20 = x_130; -x_21 = x_113; -x_22 = x_116; -x_23 = x_125; -x_24 = x_114; -x_25 = x_117; -x_26 = x_123; -x_27 = x_126; -x_28 = x_121; -x_29 = x_128; -x_30 = x_129; +x_18 = x_131; +x_19 = x_123; +x_20 = x_119; +x_21 = x_130; +x_22 = x_121; +x_23 = x_113; +x_24 = x_116; +x_25 = x_126; +x_26 = x_117; +x_27 = x_129; +x_28 = x_114; +x_29 = x_125; +x_30 = x_128; x_31 = x_134; goto block_111; } @@ -4337,7 +4337,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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_object* x_34; lean_object* x_45; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_34; lean_object* x_45; x_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); x_10 = lean_unsigned_to_nat(1u); @@ -4380,11 +4380,11 @@ goto block_44; block_33: { 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 = l_Array_append___redArg(x_19, x_21); +x_22 = l_Array_append___redArg(x_17, x_21); lean_dec_ref(x_21); -lean_inc(x_17); +lean_inc(x_20); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_17); +lean_ctor_set(x_23, 0, x_20); lean_ctor_set(x_23, 1, x_18); lean_ctor_set(x_23, 2, x_22); x_24 = l_Lean_SourceInfo_fromRef(x_11, x_5); @@ -4393,14 +4393,14 @@ x_26 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_26, 0, x_24); lean_ctor_set(x_26, 1, x_25); x_27 = l_Lake_Package_keyword; -x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_16); +x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_19); lean_dec(x_11); x_29 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_17); +lean_inc(x_20); x_30 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 0, x_20); lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_Syntax_node6(x_17, x_20, x_23, x_26, x_28, x_13, x_30, x_15); +x_31 = l_Lean_Syntax_node6(x_20, x_16, x_23, x_26, x_28, x_13, x_30, x_15); x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_31); lean_ctor_set(x_32, 1, x_3); @@ -4422,11 +4422,11 @@ x_41 = lean_ctor_get(x_34, 0); lean_inc(x_41); lean_dec_ref(x_34); x_42 = l_Array_mkArray1___redArg(x_41); -x_16 = x_36; -x_17 = x_37; +x_16 = x_38; +x_17 = x_40; x_18 = x_39; -x_19 = x_40; -x_20 = x_38; +x_19 = x_36; +x_20 = x_37; x_21 = x_42; goto block_33; } @@ -4435,11 +4435,11 @@ else lean_object* x_43; lean_dec(x_34); x_43 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_16 = x_36; -x_17 = x_37; +x_16 = x_38; +x_17 = x_40; x_18 = x_39; -x_19 = x_40; -x_20 = x_38; +x_19 = x_36; +x_20 = x_37; x_21 = x_43; goto block_33; } @@ -4589,7 +4589,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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_34; lean_object* x_45; +lean_object* x_8; lean_object* x_9; lean_object* x_10; 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_34; lean_object* x_45; x_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); x_10 = lean_unsigned_to_nat(1u); @@ -4632,12 +4632,12 @@ goto block_44; block_33: { 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 = l_Array_append___redArg(x_16, x_21); +x_22 = l_Array_append___redArg(x_19, x_21); lean_dec_ref(x_21); -lean_inc(x_19); +lean_inc(x_18); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_19); -lean_ctor_set(x_23, 1, x_17); +lean_ctor_set(x_23, 0, x_18); +lean_ctor_set(x_23, 1, x_16); lean_ctor_set(x_23, 2, x_22); x_24 = l_Lean_SourceInfo_fromRef(x_11, x_5); x_25 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__packageDataDecl__1___closed__0; @@ -4645,14 +4645,14 @@ x_26 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_26, 0, x_24); lean_ctor_set(x_26, 1, x_25); x_27 = l_Lake_Module_keyword; -x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_18); +x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_17); lean_dec(x_11); x_29 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_19); +lean_inc(x_18); x_30 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_30, 0, x_19); +lean_ctor_set(x_30, 0, x_18); lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_Syntax_node6(x_19, x_20, x_23, x_26, x_28, x_13, x_30, x_15); +x_31 = l_Lean_Syntax_node6(x_18, x_20, x_23, x_26, x_28, x_13, x_30, x_15); x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_31); lean_ctor_set(x_32, 1, x_3); @@ -4674,10 +4674,10 @@ x_41 = lean_ctor_get(x_34, 0); lean_inc(x_41); lean_dec_ref(x_34); x_42 = l_Array_mkArray1___redArg(x_41); -x_16 = x_40; -x_17 = x_39; -x_18 = x_36; -x_19 = x_37; +x_16 = x_39; +x_17 = x_36; +x_18 = x_37; +x_19 = x_40; x_20 = x_38; x_21 = x_42; goto block_33; @@ -4687,10 +4687,10 @@ else lean_object* x_43; lean_dec(x_34); x_43 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_16 = x_40; -x_17 = x_39; -x_18 = x_36; -x_19 = x_37; +x_16 = x_39; +x_17 = x_36; +x_18 = x_37; +x_19 = x_40; x_20 = x_38; x_21 = x_43; goto block_33; @@ -4858,7 +4858,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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_object* x_34; lean_object* x_45; +lean_object* x_8; lean_object* x_9; lean_object* x_10; 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_34; lean_object* x_45; x_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); x_10 = lean_unsigned_to_nat(1u); @@ -4901,12 +4901,12 @@ goto block_44; block_33: { 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 = l_Array_append___redArg(x_19, x_21); +x_22 = l_Array_append___redArg(x_18, x_21); lean_dec_ref(x_21); -lean_inc(x_17); +lean_inc(x_20); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_17); -lean_ctor_set(x_23, 1, x_18); +lean_ctor_set(x_23, 0, x_20); +lean_ctor_set(x_23, 1, x_19); lean_ctor_set(x_23, 2, x_22); x_24 = l_Lean_SourceInfo_fromRef(x_11, x_5); x_25 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__packageDataDecl__1___closed__0; @@ -4914,14 +4914,14 @@ x_26 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_26, 0, x_24); lean_ctor_set(x_26, 1, x_25); x_27 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__libraryDataDecl__1___closed__1; -x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_16); +x_28 = l_Lean_mkIdentFrom(x_11, x_27, x_17); lean_dec(x_11); x_29 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__1; -lean_inc(x_17); +lean_inc(x_20); x_30 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 0, x_20); lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_Syntax_node6(x_17, x_20, x_23, x_26, x_28, x_13, x_30, x_15); +x_31 = l_Lean_Syntax_node6(x_20, x_16, x_23, x_26, x_28, x_13, x_30, x_15); x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_31); lean_ctor_set(x_32, 1, x_3); @@ -4943,11 +4943,11 @@ x_41 = lean_ctor_get(x_34, 0); lean_inc(x_41); lean_dec_ref(x_34); x_42 = l_Array_mkArray1___redArg(x_41); -x_16 = x_36; -x_17 = x_37; -x_18 = x_39; -x_19 = x_40; -x_20 = x_38; +x_16 = x_38; +x_17 = x_36; +x_18 = x_40; +x_19 = x_39; +x_20 = x_37; x_21 = x_42; goto block_33; } @@ -4956,11 +4956,11 @@ else lean_object* x_43; lean_dec(x_34); x_43 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_16 = x_36; -x_17 = x_37; -x_18 = x_39; -x_19 = x_40; -x_20 = x_38; +x_16 = x_38; +x_17 = x_36; +x_18 = x_40; +x_19 = x_39; +x_20 = x_37; x_21 = x_43; goto block_33; } @@ -5232,13 +5232,13 @@ goto block_80; block_58: { 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; -x_29 = l_Array_append___redArg(x_27, x_28); +x_29 = l_Array_append___redArg(x_21, x_28); lean_dec_ref(x_28); -lean_inc(x_19); +lean_inc(x_27); lean_inc(x_25); x_30 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_30, 0, x_25); -lean_ctor_set(x_30, 1, x_19); +lean_ctor_set(x_30, 1, x_27); lean_ctor_set(x_30, 2, x_29); x_31 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__0; lean_inc(x_25); @@ -5260,7 +5260,7 @@ lean_ctor_set(x_38, 1, x_37); x_39 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__22; x_40 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__24; x_41 = lean_box(0); -x_42 = l_Lean_addMacroScope(x_20, x_41, x_23); +x_42 = l_Lean_addMacroScope(x_20, x_41, x_24); x_43 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__customDataDecl__1___closed__3; lean_inc(x_25); x_44 = lean_alloc_ctor(3, 4, 0); @@ -5277,11 +5277,11 @@ lean_inc(x_25); x_48 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_48, 0, x_25); lean_ctor_set(x_48, 1, x_47); -lean_inc(x_19); +lean_inc(x_27); lean_inc(x_25); -x_49 = l_Lean_Syntax_node1(x_25, x_19, x_24); +x_49 = l_Lean_Syntax_node1(x_25, x_27, x_19); lean_inc(x_25); -x_50 = l_Lean_Syntax_node3(x_25, x_19, x_22, x_48, x_49); +x_50 = l_Lean_Syntax_node3(x_25, x_27, x_18, x_48, x_49); x_51 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__builtinFacetCommand__1___lam__0___closed__28; lean_inc(x_25); x_52 = lean_alloc_ctor(2, 2, 0); @@ -5294,7 +5294,7 @@ lean_inc(x_25); x_55 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_55, 0, x_25); lean_ctor_set(x_55, 1, x_54); -x_56 = l_Lean_Syntax_node8(x_25, x_26, x_30, x_32, x_18, x_34, x_21, x_53, x_55, x_17); +x_56 = l_Lean_Syntax_node8(x_25, x_26, x_30, x_32, x_23, x_34, x_22, x_53, x_55, x_17); x_57 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_3); @@ -5338,16 +5338,16 @@ x_77 = lean_ctor_get(x_59, 0); lean_inc(x_77); lean_dec_ref(x_59); x_78 = l_Array_mkArray1___redArg(x_77); -x_18 = x_70; -x_19 = x_75; +x_18 = x_71; +x_19 = x_72; x_20 = x_60; -x_21 = x_66; -x_22 = x_71; -x_23 = x_61; -x_24 = x_72; +x_21 = x_76; +x_22 = x_66; +x_23 = x_70; +x_24 = x_61; x_25 = x_73; x_26 = x_74; -x_27 = x_76; +x_27 = x_75; x_28 = x_78; goto block_58; } @@ -5356,16 +5356,16 @@ else lean_object* x_79; lean_dec(x_59); x_79 = l_Lake___aux__Lake__Build__Data______macroRules__Lake__dataTypeDecl__1___closed__72; -x_18 = x_70; -x_19 = x_75; +x_18 = x_71; +x_19 = x_72; x_20 = x_60; -x_21 = x_66; -x_22 = x_71; -x_23 = x_61; -x_24 = x_72; +x_21 = x_76; +x_22 = x_66; +x_23 = x_70; +x_24 = x_61; x_25 = x_73; x_26 = x_74; -x_27 = x_76; +x_27 = x_75; x_28 = x_79; goto block_58; } diff --git a/stage0/stdlib/Lake/Config/Pattern.c b/stage0/stdlib/Lake/Config/Pattern.c index ae07110081d9..aee05f0e8c5b 100644 --- a/stage0/stdlib/Lake/Config/Pattern.c +++ b/stage0/stdlib/Lake/Config/Pattern.c @@ -3095,9 +3095,9 @@ goto block_52; block_44: { lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_nat_add(x_38, x_40); +x_41 = lean_nat_add(x_39, x_40); lean_dec(x_40); -lean_dec(x_38); +lean_dec(x_39); if (lean_is_scalar(x_35)) { x_42 = lean_alloc_ctor(0, 5, 0); } else { @@ -3116,7 +3116,7 @@ if (lean_is_scalar(x_25)) { lean_ctor_set(x_43, 0, x_37); lean_ctor_set(x_43, 1, x_28); lean_ctor_set(x_43, 2, x_29); -lean_ctor_set(x_43, 3, x_39); +lean_ctor_set(x_43, 3, x_38); lean_ctor_set(x_43, 4, x_42); return x_43; } @@ -3142,8 +3142,8 @@ if (lean_obj_tag(x_31) == 0) lean_object* x_50; x_50 = lean_ctor_get(x_31, 0); lean_inc(x_50); -x_38 = x_49; -x_39 = x_48; +x_38 = x_48; +x_39 = x_49; x_40 = x_50; goto block_44; } @@ -3151,8 +3151,8 @@ else { lean_object* x_51; x_51 = lean_unsigned_to_nat(0u); -x_38 = x_49; -x_39 = x_48; +x_38 = x_48; +x_39 = x_49; x_40 = x_51; goto block_44; } @@ -3569,9 +3569,9 @@ goto block_154; block_147: { lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_144 = lean_nat_add(x_141, x_143); +x_144 = lean_nat_add(x_142, x_143); lean_dec(x_143); -lean_dec(x_141); +lean_dec(x_142); if (lean_is_scalar(x_138)) { x_145 = lean_alloc_ctor(0, 5, 0); } else { @@ -3590,7 +3590,7 @@ if (lean_is_scalar(x_128)) { lean_ctor_set(x_146, 0, x_140); lean_ctor_set(x_146, 1, x_130); lean_ctor_set(x_146, 2, x_131); -lean_ctor_set(x_146, 3, x_142); +lean_ctor_set(x_146, 3, x_141); lean_ctor_set(x_146, 4, x_145); return x_146; } @@ -3616,8 +3616,8 @@ if (lean_obj_tag(x_133) == 0) lean_object* x_152; x_152 = lean_ctor_get(x_133, 0); lean_inc(x_152); -x_141 = x_151; -x_142 = x_150; +x_141 = x_150; +x_142 = x_151; x_143 = x_152; goto block_147; } @@ -3625,8 +3625,8 @@ else { lean_object* x_153; x_153 = lean_unsigned_to_nat(0u); -x_141 = x_151; -x_142 = x_150; +x_141 = x_150; +x_142 = x_151; x_143 = x_153; goto block_147; } diff --git a/stage0/stdlib/Lake/DSL/Targets.c b/stage0/stdlib/Lake/DSL/Targets.c index 706a7b890d10..12eea836e750 100644 --- a/stage0/stdlib/Lake/DSL/Targets.c +++ b/stage0/stdlib/Lake/DSL/Targets.c @@ -6915,43 +6915,43 @@ goto block_480; block_177: { 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_inc_ref(x_111); -x_132 = l_Array_append___redArg(x_111, x_131); +lean_inc_ref(x_104); +x_132 = l_Array_append___redArg(x_104, x_131); lean_dec_ref(x_131); -lean_inc(x_122); -lean_inc(x_107); +lean_inc(x_127); +lean_inc(x_125); x_133 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_133, 0, x_107); -lean_ctor_set(x_133, 1, x_122); +lean_ctor_set(x_133, 0, x_125); +lean_ctor_set(x_133, 1, x_127); lean_ctor_set(x_133, 2, x_132); -lean_inc_n(x_124, 6); -lean_inc(x_105); -lean_inc(x_107); -x_134 = l_Lean_Syntax_node7(x_107, x_105, x_133, x_124, x_124, x_124, x_124, x_124, x_124); +lean_inc_n(x_117, 6); +lean_inc(x_116); +lean_inc(x_125); +x_134 = l_Lean_Syntax_node7(x_125, x_116, x_133, x_117, x_117, x_117, x_117, x_117, x_117); x_135 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_102); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_136 = l_Lean_Name_mkStr4(x_108, x_121, x_102, x_135); -lean_inc(x_107); +lean_inc_ref(x_124); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_136 = l_Lean_Name_mkStr4(x_113, x_99, x_124, x_135); +lean_inc(x_125); x_137 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_137, 0, x_107); +lean_ctor_set(x_137, 0, x_125); lean_ctor_set(x_137, 1, x_135); x_138 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_102); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_139 = l_Lean_Name_mkStr4(x_108, x_121, x_102, x_138); +lean_inc_ref(x_124); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_139 = l_Lean_Name_mkStr4(x_113, x_99, x_124, x_138); x_140 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_141 = lean_box(2); -lean_inc(x_122); +lean_inc(x_127); x_142 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_142, 0, x_141); -lean_ctor_set(x_142, 1, x_122); +lean_ctor_set(x_142, 1, x_127); lean_ctor_set(x_142, 2, x_140); x_143 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -lean_inc(x_120); -x_144 = lean_array_push(x_143, x_120); +lean_inc(x_102); +x_144 = lean_array_push(x_143, x_102); x_145 = lean_array_push(x_144, x_142); lean_inc(x_139); x_146 = lean_alloc_ctor(1, 3, 0); @@ -6959,117 +6959,117 @@ lean_ctor_set(x_146, 0, x_141); lean_ctor_set(x_146, 1, x_139); lean_ctor_set(x_146, 2, x_145); x_147 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_102); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_148 = l_Lean_Name_mkStr4(x_108, x_121, x_102, x_147); -lean_inc_n(x_124, 2); +lean_inc_ref(x_124); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_148 = l_Lean_Name_mkStr4(x_113, x_99, x_124, x_147); +lean_inc_n(x_117, 2); lean_inc(x_148); -lean_inc(x_107); -x_149 = l_Lean_Syntax_node2(x_107, x_148, x_124, x_124); +lean_inc(x_125); +x_149 = l_Lean_Syntax_node2(x_125, x_148, x_117, x_117); x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_114); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_151 = l_Lean_Name_mkStr4(x_108, x_121, x_114, x_150); +lean_inc_ref(x_110); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_151 = l_Lean_Name_mkStr4(x_113, x_99, x_110, x_150); x_152 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__19; x_153 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__21; -lean_inc(x_104); -lean_inc(x_101); -x_154 = l_Lean_addMacroScope(x_101, x_153, x_104); -lean_inc(x_125); +lean_inc(x_103); +lean_inc(x_120); +x_154 = l_Lean_addMacroScope(x_120, x_153, x_103); +lean_inc(x_107); x_155 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_125); -lean_inc(x_118); +lean_ctor_set(x_155, 1, x_107); +lean_inc(x_128); x_156 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_118); -lean_inc(x_107); +lean_ctor_set(x_156, 1, x_128); +lean_inc(x_125); x_157 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_157, 0, x_107); +lean_ctor_set(x_157, 0, x_125); lean_ctor_set(x_157, 1, x_152); lean_ctor_set(x_157, 2, x_154); lean_ctor_set(x_157, 3, x_156); x_158 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__21; -lean_inc_ref(x_114); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_159 = l_Lean_Name_mkStr4(x_108, x_121, x_114, x_158); +lean_inc_ref(x_110); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_159 = l_Lean_Name_mkStr4(x_113, x_99, x_110, x_158); x_160 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__31; -lean_inc_ref(x_114); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_161 = l_Lean_Name_mkStr4(x_108, x_121, x_114, x_160); -lean_inc(x_107); +lean_inc_ref(x_110); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_161 = l_Lean_Name_mkStr4(x_113, x_99, x_110, x_160); +lean_inc(x_125); x_162 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_162, 0, x_107); +lean_ctor_set(x_162, 0, x_125); lean_ctor_set(x_162, 1, x_160); x_163 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__32; -lean_inc_ref(x_114); -lean_inc_ref(x_121); -lean_inc_ref(x_108); -x_164 = l_Lean_Name_mkStr4(x_108, x_121, x_114, x_163); -lean_inc(x_122); -lean_inc(x_107); -x_165 = l_Lean_Syntax_node1(x_107, x_122, x_106); +lean_inc_ref(x_110); +lean_inc_ref(x_99); +lean_inc_ref(x_113); +x_164 = l_Lean_Name_mkStr4(x_113, x_99, x_110, x_163); +lean_inc(x_127); +lean_inc(x_125); +x_165 = l_Lean_Syntax_node1(x_125, x_127, x_122); x_166 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__33; -lean_inc(x_107); +lean_inc(x_125); x_167 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_167, 0, x_107); +lean_ctor_set(x_167, 0, x_125); lean_ctor_set(x_167, 1, x_166); -lean_inc(x_124); -lean_inc(x_107); -x_168 = l_Lean_Syntax_node4(x_107, x_164, x_165, x_124, x_167, x_126); -lean_inc(x_107); -x_169 = l_Lean_Syntax_node2(x_107, x_161, x_162, x_168); -lean_inc(x_107); -x_170 = l_Lean_Syntax_node3(x_107, x_159, x_109, x_169, x_129); -lean_inc(x_122); -lean_inc(x_107); -x_171 = l_Lean_Syntax_node4(x_107, x_122, x_127, x_100, x_123, x_170); -lean_inc(x_107); -x_172 = l_Lean_Syntax_node2(x_107, x_151, x_157, x_171); -lean_inc_n(x_124, 2); -lean_inc(x_107); -x_173 = l_Lean_Syntax_node2(x_107, x_103, x_124, x_124); -if (lean_obj_tag(x_117) == 1) +lean_inc(x_117); +lean_inc(x_125); +x_168 = l_Lean_Syntax_node4(x_125, x_164, x_165, x_117, x_167, x_108); +lean_inc(x_125); +x_169 = l_Lean_Syntax_node2(x_125, x_161, x_162, x_168); +lean_inc(x_125); +x_170 = l_Lean_Syntax_node3(x_125, x_159, x_129, x_169, x_109); +lean_inc(x_127); +lean_inc(x_125); +x_171 = l_Lean_Syntax_node4(x_125, x_127, x_105, x_119, x_111, x_170); +lean_inc(x_125); +x_172 = l_Lean_Syntax_node2(x_125, x_151, x_157, x_171); +lean_inc_n(x_117, 2); +lean_inc(x_125); +x_173 = l_Lean_Syntax_node2(x_125, x_121, x_117, x_117); +if (lean_obj_tag(x_118) == 1) { lean_object* x_174; lean_object* x_175; -x_174 = lean_ctor_get(x_117, 0); +x_174 = lean_ctor_get(x_118, 0); lean_inc(x_174); -lean_dec_ref(x_117); +lean_dec_ref(x_118); x_175 = l_Array_mkArray1___redArg(x_174); x_4 = x_99; -x_5 = x_101; -x_6 = x_102; -x_7 = x_104; -x_8 = x_148; -x_9 = x_105; -x_10 = x_172; -x_11 = x_107; -x_12 = x_137; -x_13 = x_108; -x_14 = x_110; -x_15 = x_111; -x_16 = x_136; +x_5 = x_172; +x_6 = x_100; +x_7 = x_101; +x_8 = x_137; +x_9 = x_102; +x_10 = x_103; +x_11 = x_104; +x_12 = x_106; +x_13 = x_107; +x_14 = x_139; +x_15 = x_149; +x_16 = x_110; x_17 = x_112; x_18 = x_173; -x_19 = x_146; -x_20 = x_113; +x_19 = x_113; +x_20 = x_148; x_21 = x_114; x_22 = x_115; -x_23 = x_116; -x_24 = x_134; -x_25 = x_118; -x_26 = x_120; -x_27 = x_119; -x_28 = x_122; -x_29 = x_121; -x_30 = x_139; -x_31 = x_124; -x_32 = x_125; -x_33 = x_149; +x_23 = x_146; +x_24 = x_116; +x_25 = x_136; +x_26 = x_117; +x_27 = x_134; +x_28 = x_120; +x_29 = x_123; +x_30 = x_124; +x_31 = x_125; +x_32 = x_126; +x_33 = x_127; x_34 = x_128; x_35 = x_130; x_36 = x_175; @@ -7078,38 +7078,38 @@ goto block_89; else { lean_object* x_176; -lean_dec(x_117); +lean_dec(x_118); x_176 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; x_4 = x_99; -x_5 = x_101; -x_6 = x_102; -x_7 = x_104; -x_8 = x_148; -x_9 = x_105; -x_10 = x_172; -x_11 = x_107; -x_12 = x_137; -x_13 = x_108; -x_14 = x_110; -x_15 = x_111; -x_16 = x_136; +x_5 = x_172; +x_6 = x_100; +x_7 = x_101; +x_8 = x_137; +x_9 = x_102; +x_10 = x_103; +x_11 = x_104; +x_12 = x_106; +x_13 = x_107; +x_14 = x_139; +x_15 = x_149; +x_16 = x_110; x_17 = x_112; x_18 = x_173; -x_19 = x_146; -x_20 = x_113; +x_19 = x_113; +x_20 = x_148; x_21 = x_114; x_22 = x_115; -x_23 = x_116; -x_24 = x_134; -x_25 = x_118; -x_26 = x_120; -x_27 = x_119; -x_28 = x_122; -x_29 = x_121; -x_30 = x_139; -x_31 = x_124; -x_32 = x_125; -x_33 = x_149; +x_23 = x_146; +x_24 = x_116; +x_25 = x_136; +x_26 = x_117; +x_27 = x_134; +x_28 = x_120; +x_29 = x_123; +x_30 = x_124; +x_31 = x_125; +x_32 = x_126; +x_33 = x_127; x_34 = x_128; x_35 = x_130; x_36 = x_176; @@ -7133,7 +7133,7 @@ lean_inc(x_199); lean_inc(x_197); lean_inc(x_196); lean_ctor_set(x_193, 5, x_199); -x_200 = l_Lake_DSL_expandOptSimpleBinder(x_179, x_193, x_194); +x_200 = l_Lake_DSL_expandOptSimpleBinder(x_181, x_193, x_194); if (lean_obj_tag(x_200) == 0) { lean_object* x_201; lean_object* x_202; uint8_t 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; @@ -7146,15 +7146,15 @@ x_203 = 0; x_204 = l_Lean_SourceInfo_fromRef(x_199, x_203); lean_dec(x_199); x_205 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__42; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_206 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_205); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_206 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_205); x_207 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__43; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_208 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_207); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_208 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_207); x_209 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_210 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; lean_inc(x_204); @@ -7167,9 +7167,9 @@ lean_inc(x_204); x_212 = l_Lean_Syntax_node1(x_204, x_208, x_211); x_213 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__47; x_214 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__48; -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_215 = l_Lean_Name_mkStr4(x_186, x_185, x_213, x_214); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_215 = l_Lean_Name_mkStr4(x_189, x_179, x_213, x_214); x_216 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_217 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; lean_inc(x_197); @@ -7189,12 +7189,12 @@ lean_inc(x_204); x_222 = l_Lean_Syntax_node2(x_204, x_206, x_212, x_221); x_223 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__53; x_224 = lean_array_push(x_223, x_222); -x_225 = l_Lake_DSL_expandAttrs(x_189); +x_225 = l_Lake_DSL_expandAttrs(x_190); x_226 = l_Array_append___redArg(x_224, x_225); lean_dec_ref(x_225); -x_227 = l_Lean_TSyntax_getId(x_184); -lean_inc(x_184); -x_228 = l_Lake_Name_quoteFrom(x_184, x_227, x_203); +x_227 = l_Lean_TSyntax_getId(x_182); +lean_inc(x_182); +x_228 = l_Lake_Name_quoteFrom(x_182, x_227, x_203); x_229 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; x_230 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; lean_inc(x_204); @@ -7219,15 +7219,15 @@ lean_ctor_set(x_238, 1, x_234); lean_ctor_set(x_238, 2, x_236); lean_ctor_set(x_238, 3, x_237); x_239 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_240 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_239); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_240 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_239); x_241 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_242 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_241); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_242 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_241); x_243 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; lean_inc(x_204); x_244 = lean_alloc_ctor(2, 2, 0); @@ -7240,29 +7240,29 @@ lean_inc(x_197); lean_inc(x_196); x_248 = l_Lean_addMacroScope(x_196, x_247, x_197); x_249 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_250 = l_Lean_Name_mkStr3(x_186, x_185, x_181); +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_250 = l_Lean_Name_mkStr3(x_189, x_179, x_187); x_251 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_251, 0, x_250); x_252 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_181); -lean_inc_ref(x_186); -x_253 = l_Lean_Name_mkStr3(x_186, x_252, x_181); +lean_inc_ref(x_187); +lean_inc_ref(x_189); +x_253 = l_Lean_Name_mkStr3(x_189, x_252, x_187); x_254 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_254, 0, x_253); -lean_inc_ref(x_186); -x_255 = l_Lean_Name_mkStr2(x_186, x_252); +lean_inc_ref(x_189); +x_255 = l_Lean_Name_mkStr2(x_189, x_252); x_256 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_256, 0, x_255); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_257 = l_Lean_Name_mkStr2(x_186, x_185); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_257 = l_Lean_Name_mkStr2(x_189, x_179); x_258 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_258, 0, x_257); -lean_inc_ref(x_186); -x_259 = l_Lean_Name_mkStr1(x_186); +lean_inc_ref(x_189); +x_259 = l_Lean_Name_mkStr1(x_189); x_260 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_260, 0, x_259); x_261 = lean_alloc_ctor(1, 2, 0); @@ -7326,102 +7326,102 @@ lean_inc(x_204); x_282 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_282, 0, x_204); lean_ctor_set(x_282, 1, x_281); -lean_inc(x_187); +lean_inc(x_183); lean_inc_ref(x_282); lean_inc_ref(x_233); -lean_inc(x_184); +lean_inc(x_182); lean_inc_ref(x_211); lean_inc(x_204); -x_283 = l_Lean_Syntax_node8(x_204, x_229, x_211, x_231, x_184, x_233, x_238, x_280, x_282, x_187); +x_283 = l_Lean_Syntax_node8(x_204, x_229, x_211, x_231, x_182, x_233, x_238, x_280, x_282, x_183); x_284 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_285 = l_Lean_Name_mkStr4(x_186, x_185, x_181, x_284); +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_285 = l_Lean_Name_mkStr4(x_189, x_179, x_187, x_284); x_286 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_287 = l_Lean_Name_mkStr4(x_186, x_185, x_181, x_286); -if (lean_obj_tag(x_183) == 1) +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_287 = l_Lean_Name_mkStr4(x_189, x_179, x_187, x_286); +if (lean_obj_tag(x_188) == 1) { lean_object* x_288; lean_object* x_289; -x_288 = lean_ctor_get(x_183, 0); +x_288 = lean_ctor_get(x_188, 0); lean_inc(x_288); -lean_dec_ref(x_183); +lean_dec_ref(x_188); x_289 = l_Array_mkArray1___redArg(x_288); -x_99 = x_180; -x_100 = x_273; -x_101 = x_196; -x_102 = x_181; -x_103 = x_182; -x_104 = x_197; -x_105 = x_287; -x_106 = x_201; -x_107 = x_204; -x_108 = x_186; -x_109 = x_269; -x_110 = x_226; -x_111 = x_210; -x_112 = x_283; -x_113 = x_233; +x_99 = x_179; +x_100 = x_282; +x_101 = x_180; +x_102 = x_182; +x_103 = x_197; +x_104 = x_210; +x_105 = x_183; +x_106 = x_226; +x_107 = x_219; +x_108 = x_185; +x_109 = x_279; +x_110 = x_186; +x_111 = x_228; +x_112 = x_285; +x_113 = x_189; x_114 = x_191; -x_115 = x_202; -x_116 = x_285; -x_117 = x_192; -x_118 = x_219; -x_119 = x_282; -x_120 = x_184; -x_121 = x_185; -x_122 = x_209; -x_123 = x_228; -x_124 = x_211; -x_125 = x_219; -x_126 = x_188; -x_127 = x_187; -x_128 = x_190; -x_129 = x_279; -x_130 = x_274; +x_115 = x_274; +x_116 = x_287; +x_117 = x_211; +x_118 = x_192; +x_119 = x_273; +x_120 = x_196; +x_121 = x_184; +x_122 = x_201; +x_123 = x_202; +x_124 = x_187; +x_125 = x_204; +x_126 = x_233; +x_127 = x_209; +x_128 = x_219; +x_129 = x_269; +x_130 = x_283; x_131 = x_289; goto block_177; } else { lean_object* x_290; -lean_dec(x_183); +lean_dec(x_188); x_290 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_99 = x_180; -x_100 = x_273; -x_101 = x_196; -x_102 = x_181; -x_103 = x_182; -x_104 = x_197; -x_105 = x_287; -x_106 = x_201; -x_107 = x_204; -x_108 = x_186; -x_109 = x_269; -x_110 = x_226; -x_111 = x_210; -x_112 = x_283; -x_113 = x_233; +x_99 = x_179; +x_100 = x_282; +x_101 = x_180; +x_102 = x_182; +x_103 = x_197; +x_104 = x_210; +x_105 = x_183; +x_106 = x_226; +x_107 = x_219; +x_108 = x_185; +x_109 = x_279; +x_110 = x_186; +x_111 = x_228; +x_112 = x_285; +x_113 = x_189; x_114 = x_191; -x_115 = x_202; -x_116 = x_285; -x_117 = x_192; -x_118 = x_219; -x_119 = x_282; -x_120 = x_184; -x_121 = x_185; -x_122 = x_209; -x_123 = x_228; -x_124 = x_211; -x_125 = x_219; -x_126 = x_188; -x_127 = x_187; -x_128 = x_190; -x_129 = x_279; -x_130 = x_274; +x_115 = x_274; +x_116 = x_287; +x_117 = x_211; +x_118 = x_192; +x_119 = x_273; +x_120 = x_196; +x_121 = x_184; +x_122 = x_201; +x_123 = x_202; +x_124 = x_187; +x_125 = x_204; +x_126 = x_233; +x_127 = x_209; +x_128 = x_219; +x_129 = x_269; +x_130 = x_283; x_131 = x_290; goto block_177; } @@ -7433,18 +7433,18 @@ lean_dec(x_199); lean_dec(x_197); lean_dec(x_196); lean_dec(x_192); -lean_dec_ref(x_191); +lean_dec(x_191); lean_dec(x_190); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec(x_188); -lean_dec(x_187); +lean_dec_ref(x_187); lean_dec_ref(x_186); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); lean_dec(x_183); lean_dec(x_182); -lean_dec_ref(x_181); lean_dec(x_180); +lean_dec_ref(x_179); x_291 = !lean_is_exclusive(x_200); if (x_291 == 0) { @@ -7494,7 +7494,7 @@ lean_ctor_set(x_302, 2, x_297); lean_ctor_set(x_302, 3, x_298); lean_ctor_set(x_302, 4, x_299); lean_ctor_set(x_302, 5, x_301); -x_303 = l_Lake_DSL_expandOptSimpleBinder(x_179, x_302, x_194); +x_303 = l_Lake_DSL_expandOptSimpleBinder(x_181, x_302, x_194); if (lean_obj_tag(x_303) == 0) { lean_object* x_304; lean_object* x_305; uint8_t 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; @@ -7507,15 +7507,15 @@ x_306 = 0; x_307 = l_Lean_SourceInfo_fromRef(x_301, x_306); lean_dec(x_301); x_308 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__42; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_309 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_308); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_309 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_308); x_310 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__43; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_311 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_310); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_311 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_310); x_312 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_313 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; lean_inc(x_307); @@ -7528,9 +7528,9 @@ lean_inc(x_307); x_315 = l_Lean_Syntax_node1(x_307, x_311, x_314); x_316 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__47; x_317 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__48; -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_318 = l_Lean_Name_mkStr4(x_186, x_185, x_316, x_317); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_318 = l_Lean_Name_mkStr4(x_189, x_179, x_316, x_317); x_319 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_320 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; lean_inc(x_297); @@ -7550,12 +7550,12 @@ lean_inc(x_307); x_325 = l_Lean_Syntax_node2(x_307, x_309, x_315, x_324); x_326 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__53; x_327 = lean_array_push(x_326, x_325); -x_328 = l_Lake_DSL_expandAttrs(x_189); +x_328 = l_Lake_DSL_expandAttrs(x_190); x_329 = l_Array_append___redArg(x_327, x_328); lean_dec_ref(x_328); -x_330 = l_Lean_TSyntax_getId(x_184); -lean_inc(x_184); -x_331 = l_Lake_Name_quoteFrom(x_184, x_330, x_306); +x_330 = l_Lean_TSyntax_getId(x_182); +lean_inc(x_182); +x_331 = l_Lake_Name_quoteFrom(x_182, x_330, x_306); x_332 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; x_333 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; lean_inc(x_307); @@ -7580,15 +7580,15 @@ lean_ctor_set(x_341, 1, x_337); lean_ctor_set(x_341, 2, x_339); lean_ctor_set(x_341, 3, x_340); x_342 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_343 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_342); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_343 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_342); x_344 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_191); -lean_inc_ref(x_185); lean_inc_ref(x_186); -x_345 = l_Lean_Name_mkStr4(x_186, x_185, x_191, x_344); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_345 = l_Lean_Name_mkStr4(x_189, x_179, x_186, x_344); x_346 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; lean_inc(x_307); x_347 = lean_alloc_ctor(2, 2, 0); @@ -7601,29 +7601,29 @@ lean_inc(x_297); lean_inc(x_296); x_351 = l_Lean_addMacroScope(x_296, x_350, x_297); x_352 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_353 = l_Lean_Name_mkStr3(x_186, x_185, x_181); +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_353 = l_Lean_Name_mkStr3(x_189, x_179, x_187); x_354 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_354, 0, x_353); x_355 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_181); -lean_inc_ref(x_186); -x_356 = l_Lean_Name_mkStr3(x_186, x_355, x_181); +lean_inc_ref(x_187); +lean_inc_ref(x_189); +x_356 = l_Lean_Name_mkStr3(x_189, x_355, x_187); x_357 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_357, 0, x_356); -lean_inc_ref(x_186); -x_358 = l_Lean_Name_mkStr2(x_186, x_355); +lean_inc_ref(x_189); +x_358 = l_Lean_Name_mkStr2(x_189, x_355); x_359 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_359, 0, x_358); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_360 = l_Lean_Name_mkStr2(x_186, x_185); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_360 = l_Lean_Name_mkStr2(x_189, x_179); x_361 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_361, 0, x_360); -lean_inc_ref(x_186); -x_362 = l_Lean_Name_mkStr1(x_186); +lean_inc_ref(x_189); +x_362 = l_Lean_Name_mkStr1(x_189); x_363 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_363, 0, x_362); x_364 = lean_alloc_ctor(1, 2, 0); @@ -7687,102 +7687,102 @@ lean_inc(x_307); x_385 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_385, 0, x_307); lean_ctor_set(x_385, 1, x_384); -lean_inc(x_187); +lean_inc(x_183); lean_inc_ref(x_385); lean_inc_ref(x_336); -lean_inc(x_184); +lean_inc(x_182); lean_inc_ref(x_314); lean_inc(x_307); -x_386 = l_Lean_Syntax_node8(x_307, x_332, x_314, x_334, x_184, x_336, x_341, x_383, x_385, x_187); +x_386 = l_Lean_Syntax_node8(x_307, x_332, x_314, x_334, x_182, x_336, x_341, x_383, x_385, x_183); x_387 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_388 = l_Lean_Name_mkStr4(x_186, x_185, x_181, x_387); +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_388 = l_Lean_Name_mkStr4(x_189, x_179, x_187, x_387); x_389 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_181); -lean_inc_ref(x_185); -lean_inc_ref(x_186); -x_390 = l_Lean_Name_mkStr4(x_186, x_185, x_181, x_389); -if (lean_obj_tag(x_183) == 1) +lean_inc_ref(x_187); +lean_inc_ref(x_179); +lean_inc_ref(x_189); +x_390 = l_Lean_Name_mkStr4(x_189, x_179, x_187, x_389); +if (lean_obj_tag(x_188) == 1) { lean_object* x_391; lean_object* x_392; -x_391 = lean_ctor_get(x_183, 0); +x_391 = lean_ctor_get(x_188, 0); lean_inc(x_391); -lean_dec_ref(x_183); +lean_dec_ref(x_188); x_392 = l_Array_mkArray1___redArg(x_391); -x_99 = x_180; -x_100 = x_376; -x_101 = x_296; -x_102 = x_181; -x_103 = x_182; -x_104 = x_297; -x_105 = x_390; -x_106 = x_304; -x_107 = x_307; -x_108 = x_186; -x_109 = x_372; -x_110 = x_329; -x_111 = x_313; -x_112 = x_386; -x_113 = x_336; +x_99 = x_179; +x_100 = x_385; +x_101 = x_180; +x_102 = x_182; +x_103 = x_297; +x_104 = x_313; +x_105 = x_183; +x_106 = x_329; +x_107 = x_322; +x_108 = x_185; +x_109 = x_382; +x_110 = x_186; +x_111 = x_331; +x_112 = x_388; +x_113 = x_189; x_114 = x_191; -x_115 = x_305; -x_116 = x_388; -x_117 = x_192; -x_118 = x_322; -x_119 = x_385; -x_120 = x_184; -x_121 = x_185; -x_122 = x_312; -x_123 = x_331; -x_124 = x_314; -x_125 = x_322; -x_126 = x_188; -x_127 = x_187; -x_128 = x_190; -x_129 = x_382; -x_130 = x_377; +x_115 = x_377; +x_116 = x_390; +x_117 = x_314; +x_118 = x_192; +x_119 = x_376; +x_120 = x_296; +x_121 = x_184; +x_122 = x_304; +x_123 = x_305; +x_124 = x_187; +x_125 = x_307; +x_126 = x_336; +x_127 = x_312; +x_128 = x_322; +x_129 = x_372; +x_130 = x_386; x_131 = x_392; goto block_177; } else { lean_object* x_393; -lean_dec(x_183); +lean_dec(x_188); x_393 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_99 = x_180; -x_100 = x_376; -x_101 = x_296; -x_102 = x_181; -x_103 = x_182; -x_104 = x_297; -x_105 = x_390; -x_106 = x_304; -x_107 = x_307; -x_108 = x_186; -x_109 = x_372; -x_110 = x_329; -x_111 = x_313; -x_112 = x_386; -x_113 = x_336; +x_99 = x_179; +x_100 = x_385; +x_101 = x_180; +x_102 = x_182; +x_103 = x_297; +x_104 = x_313; +x_105 = x_183; +x_106 = x_329; +x_107 = x_322; +x_108 = x_185; +x_109 = x_382; +x_110 = x_186; +x_111 = x_331; +x_112 = x_388; +x_113 = x_189; x_114 = x_191; -x_115 = x_305; -x_116 = x_388; -x_117 = x_192; -x_118 = x_322; -x_119 = x_385; -x_120 = x_184; -x_121 = x_185; -x_122 = x_312; -x_123 = x_331; -x_124 = x_314; -x_125 = x_322; -x_126 = x_188; -x_127 = x_187; -x_128 = x_190; -x_129 = x_382; -x_130 = x_377; +x_115 = x_377; +x_116 = x_390; +x_117 = x_314; +x_118 = x_192; +x_119 = x_376; +x_120 = x_296; +x_121 = x_184; +x_122 = x_304; +x_123 = x_305; +x_124 = x_187; +x_125 = x_307; +x_126 = x_336; +x_127 = x_312; +x_128 = x_322; +x_129 = x_372; +x_130 = x_386; x_131 = x_393; goto block_177; } @@ -7794,18 +7794,18 @@ lean_dec(x_301); lean_dec(x_297); lean_dec(x_296); lean_dec(x_192); -lean_dec_ref(x_191); +lean_dec(x_191); lean_dec(x_190); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec(x_188); -lean_dec(x_187); +lean_dec_ref(x_187); lean_dec_ref(x_186); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); lean_dec(x_183); lean_dec(x_182); -lean_dec_ref(x_181); lean_dec(x_180); +lean_dec_ref(x_179); x_394 = lean_ctor_get(x_303, 0); lean_inc(x_394); x_395 = lean_ctor_get(x_303, 1); @@ -8001,19 +8001,19 @@ lean_object* x_446; lean_dec(x_400); x_446 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_446, 0, x_441); -x_179 = x_404; +x_179 = x_409; x_180 = x_417; -x_181 = x_416; -x_182 = x_422; -x_183 = x_401; -x_184 = x_402; -x_185 = x_409; -x_186 = x_408; -x_187 = x_434; -x_188 = x_435; -x_189 = x_403; -x_190 = x_411; -x_191 = x_410; +x_181 = x_404; +x_182 = x_401; +x_183 = x_434; +x_184 = x_422; +x_185 = x_435; +x_186 = x_410; +x_187 = x_416; +x_188 = x_402; +x_189 = x_408; +x_190 = x_403; +x_191 = x_411; x_192 = x_446; x_193 = x_405; x_194 = x_406; @@ -8027,19 +8027,19 @@ lean_object* x_447; lean_dec(x_436); lean_dec(x_400); x_447 = lean_box(0); -x_179 = x_404; +x_179 = x_409; x_180 = x_417; -x_181 = x_416; -x_182 = x_422; -x_183 = x_401; -x_184 = x_402; -x_185 = x_409; -x_186 = x_408; -x_187 = x_434; -x_188 = x_435; -x_189 = x_403; -x_190 = x_411; -x_191 = x_410; +x_181 = x_404; +x_182 = x_401; +x_183 = x_434; +x_184 = x_422; +x_185 = x_435; +x_186 = x_410; +x_187 = x_416; +x_188 = x_402; +x_189 = x_408; +x_190 = x_403; +x_191 = x_411; x_192 = x_447; x_193 = x_405; x_194 = x_406; @@ -8136,8 +8136,8 @@ x_470 = l_Lean_Syntax_getArg(x_465, x_94); lean_dec(x_465); x_471 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_471, 0, x_470); -x_401 = x_451; -x_402 = x_460; +x_401 = x_460; +x_402 = x_451; x_403 = x_450; x_404 = x_471; x_405 = x_2; @@ -8150,8 +8150,8 @@ else lean_object* x_472; lean_dec(x_465); x_472 = lean_box(0); -x_401 = x_451; -x_402 = x_460; +x_401 = x_460; +x_402 = x_451; x_403 = x_450; x_404 = x_472; x_405 = x_2; @@ -8203,142 +8203,142 @@ goto block_473; block_89: { 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_inc_ref(x_15); -x_37 = l_Array_append___redArg(x_15, x_36); +lean_inc_ref(x_11); +x_37 = l_Array_append___redArg(x_11, x_36); lean_dec_ref(x_36); -lean_inc(x_28); -lean_inc(x_11); +lean_inc(x_33); +lean_inc(x_31); x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_11); -lean_ctor_set(x_38, 1, x_28); +lean_ctor_set(x_38, 0, x_31); +lean_ctor_set(x_38, 1, x_33); lean_ctor_set(x_38, 2, x_37); lean_inc(x_18); -lean_inc(x_27); -lean_inc(x_4); -lean_inc(x_11); -x_39 = l_Lean_Syntax_node4(x_11, x_4, x_27, x_10, x_18, x_38); -lean_inc(x_11); -x_40 = l_Lean_Syntax_node4(x_11, x_16, x_12, x_19, x_33, x_39); -lean_inc(x_23); -lean_inc(x_11); -x_41 = l_Lean_Syntax_node2(x_11, x_23, x_24, x_40); +lean_inc(x_6); +lean_inc(x_7); +lean_inc(x_31); +x_39 = l_Lean_Syntax_node4(x_31, x_7, x_6, x_5, x_18, x_38); +lean_inc(x_31); +x_40 = l_Lean_Syntax_node4(x_31, x_25, x_8, x_23, x_15, x_39); +lean_inc(x_17); +lean_inc(x_31); +x_41 = l_Lean_Syntax_node2(x_31, x_17, x_27, x_40); x_42 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_21); -lean_inc_ref(x_29); -lean_inc_ref(x_13); -x_43 = l_Lean_Name_mkStr4(x_13, x_29, x_21, x_42); +lean_inc_ref(x_16); +lean_inc_ref(x_4); +lean_inc_ref(x_19); +x_43 = l_Lean_Name_mkStr4(x_19, x_4, x_16, x_42); x_44 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_11); +lean_inc(x_31); x_45 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_45, 0, x_11); +lean_ctor_set(x_45, 0, x_31); lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_Syntax_SepArray_ofElems(x_35, x_14); -lean_dec_ref(x_14); -x_47 = l_Array_append___redArg(x_15, x_46); +x_46 = l_Lean_Syntax_SepArray_ofElems(x_22, x_12); +lean_dec_ref(x_12); +x_47 = l_Array_append___redArg(x_11, x_46); lean_dec_ref(x_46); -lean_inc(x_28); -lean_inc(x_11); +lean_inc(x_33); +lean_inc(x_31); x_48 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_48, 0, x_11); -lean_ctor_set(x_48, 1, x_28); +lean_ctor_set(x_48, 0, x_31); +lean_ctor_set(x_48, 1, x_33); lean_ctor_set(x_48, 2, x_47); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_11); +lean_inc(x_31); x_50 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_50, 0, x_11); +lean_ctor_set(x_50, 0, x_31); lean_ctor_set(x_50, 1, x_49); -lean_inc(x_11); -x_51 = l_Lean_Syntax_node3(x_11, x_43, x_45, x_48, x_50); -lean_inc(x_28); -lean_inc(x_11); -x_52 = l_Lean_Syntax_node1(x_11, x_28, x_51); -lean_inc_n(x_31, 6); -lean_inc(x_11); -x_53 = l_Lean_Syntax_node7(x_11, x_9, x_31, x_52, x_31, x_31, x_31, x_31, x_31); +lean_inc(x_31); +x_51 = l_Lean_Syntax_node3(x_31, x_43, x_45, x_48, x_50); +lean_inc(x_33); +lean_inc(x_31); +x_52 = l_Lean_Syntax_node1(x_31, x_33, x_51); +lean_inc_n(x_26, 6); +lean_inc(x_31); +x_53 = l_Lean_Syntax_node7(x_31, x_24, x_26, x_52, x_26, x_26, x_26, x_26, x_26); x_54 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_29); -lean_inc_ref(x_13); -x_55 = l_Lean_Name_mkStr4(x_13, x_29, x_6, x_54); +lean_inc_ref(x_4); +lean_inc_ref(x_19); +x_55 = l_Lean_Name_mkStr4(x_19, x_4, x_30, x_54); x_56 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_11); +lean_inc(x_31); x_57 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_57, 0, x_11); +lean_ctor_set(x_57, 0, x_31); lean_ctor_set(x_57, 1, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_59 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_7); -lean_inc(x_5); -x_60 = l_Lean_addMacroScope(x_5, x_59, x_7); -lean_inc(x_25); -lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_28); +x_60 = l_Lean_addMacroScope(x_28, x_59, x_10); +lean_inc(x_34); +lean_inc(x_31); x_61 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_61, 0, x_11); +lean_ctor_set(x_61, 0, x_31); lean_ctor_set(x_61, 1, x_58); lean_ctor_set(x_61, 2, x_60); -lean_ctor_set(x_61, 3, x_25); +lean_ctor_set(x_61, 3, x_34); +lean_inc(x_26); lean_inc(x_31); -lean_inc(x_11); -x_62 = l_Lean_Syntax_node2(x_11, x_30, x_61, x_31); +x_62 = l_Lean_Syntax_node2(x_31, x_14, x_61, x_26); x_63 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_64 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_7); -lean_inc(x_5); -x_65 = l_Lean_addMacroScope(x_5, x_64, x_7); +lean_inc(x_10); +lean_inc(x_28); +x_65 = l_Lean_addMacroScope(x_28, x_64, x_10); x_66 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__8; x_67 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_32); +lean_ctor_set(x_67, 1, x_13); x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__9; -lean_inc(x_25); +lean_inc(x_34); x_69 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_25); +lean_ctor_set(x_69, 1, x_34); x_70 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_70, 0, x_67); lean_ctor_set(x_70, 1, x_69); -lean_inc(x_11); +lean_inc(x_31); x_71 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_71, 0, x_11); +lean_ctor_set(x_71, 0, x_31); lean_ctor_set(x_71, 1, x_63); lean_ctor_set(x_71, 2, x_65); lean_ctor_set(x_71, 3, x_70); -lean_inc(x_11); -x_72 = l_Lean_Syntax_node2(x_11, x_34, x_20, x_71); -lean_inc(x_28); -lean_inc(x_11); -x_73 = l_Lean_Syntax_node1(x_11, x_28, x_72); lean_inc(x_31); -lean_inc(x_11); -x_74 = l_Lean_Syntax_node2(x_11, x_8, x_31, x_73); +x_72 = l_Lean_Syntax_node2(x_31, x_21, x_32, x_71); +lean_inc(x_33); +lean_inc(x_31); +x_73 = l_Lean_Syntax_node1(x_31, x_33, x_72); +lean_inc(x_26); +lean_inc(x_31); +x_74 = l_Lean_Syntax_node2(x_31, x_20, x_26, x_73); x_75 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_76 = l_Lean_Name_mkStr4(x_13, x_29, x_21, x_75); +x_76 = l_Lean_Name_mkStr4(x_19, x_4, x_16, x_75); x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_11); +lean_inc(x_31); x_78 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_78, 0, x_11); +lean_ctor_set(x_78, 0, x_31); lean_ctor_set(x_78, 1, x_77); x_79 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_80 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_81 = l_Lean_addMacroScope(x_5, x_80, x_7); -lean_inc(x_11); +x_81 = l_Lean_addMacroScope(x_28, x_80, x_10); +lean_inc(x_31); x_82 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_82, 0, x_11); +lean_ctor_set(x_82, 0, x_31); lean_ctor_set(x_82, 1, x_79); lean_ctor_set(x_82, 2, x_81); -lean_ctor_set(x_82, 3, x_25); -lean_inc(x_11); -x_83 = l_Lean_Syntax_node3(x_11, x_76, x_26, x_78, x_82); +lean_ctor_set(x_82, 3, x_34); lean_inc(x_31); -lean_inc(x_11); -x_84 = l_Lean_Syntax_node4(x_11, x_4, x_27, x_83, x_18, x_31); -lean_inc(x_11); -x_85 = l_Lean_Syntax_node5(x_11, x_55, x_57, x_62, x_74, x_84, x_31); -lean_inc(x_11); -x_86 = l_Lean_Syntax_node2(x_11, x_23, x_53, x_85); -x_87 = l_Lean_Syntax_node3(x_11, x_28, x_17, x_41, x_86); +x_83 = l_Lean_Syntax_node3(x_31, x_76, x_9, x_78, x_82); +lean_inc(x_26); +lean_inc(x_31); +x_84 = l_Lean_Syntax_node4(x_31, x_7, x_6, x_83, x_18, x_26); +lean_inc(x_31); +x_85 = l_Lean_Syntax_node5(x_31, x_55, x_57, x_62, x_74, x_84, x_26); +lean_inc(x_31); +x_86 = l_Lean_Syntax_node2(x_31, x_17, x_53, x_85); +x_87 = l_Lean_Syntax_node3(x_31, x_33, x_35, x_41, 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_22); +lean_ctor_set(x_88, 1, x_29); return x_88; } } @@ -8808,22 +8808,22 @@ lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; x_281 = lean_ctor_get(x_280, 0); lean_inc(x_281); lean_dec_ref(x_280); -lean_inc_ref(x_270); -lean_inc(x_260); -lean_inc(x_257); +lean_inc_ref(x_269); +lean_inc(x_264); +lean_inc(x_261); x_282 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_282, 0, x_257); -lean_ctor_set(x_282, 1, x_260); -lean_ctor_set(x_282, 2, x_270); +lean_ctor_set(x_282, 0, x_261); +lean_ctor_set(x_282, 1, x_264); +lean_ctor_set(x_282, 2, x_269); lean_inc_ref(x_282); -lean_inc(x_257); -x_283 = l_Lean_Syntax_node1(x_257, x_265, x_282); -lean_inc(x_257); -x_284 = l_Lean_Syntax_node2(x_257, x_261, x_268, x_282); -x_285 = l_Lean_Syntax_node2(x_257, x_262, x_283, x_284); +lean_inc(x_261); +x_283 = l_Lean_Syntax_node1(x_261, x_265, x_282); +lean_inc(x_261); +x_284 = l_Lean_Syntax_node2(x_261, x_271, x_257, x_282); +x_285 = l_Lean_Syntax_node2(x_261, x_267, x_283, x_284); x_286 = lean_unsigned_to_nat(2u); x_287 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_288 = lean_array_push(x_287, x_271); +x_288 = lean_array_push(x_287, x_266); x_289 = lean_array_push(x_288, x_285); x_290 = l_Lake_DSL_expandAttrs(x_7); x_291 = l_Array_append___redArg(x_289, x_290); @@ -8840,21 +8840,21 @@ lean_object* x_295; x_295 = lean_ctor_get(x_294, 0); lean_inc(x_295); lean_dec_ref(x_294); -x_133 = x_258; -x_134 = x_275; +x_133 = x_292; +x_134 = x_258; x_135 = x_259; -x_136 = x_292; -x_137 = x_260; -x_138 = x_279; -x_139 = x_263; -x_140 = x_264; -x_141 = x_291; -x_142 = x_286; -x_143 = x_267; -x_144 = x_266; -x_145 = x_270; -x_146 = x_269; -x_147 = x_281; +x_136 = x_291; +x_137 = x_279; +x_138 = x_281; +x_139 = x_286; +x_140 = x_260; +x_141 = x_262; +x_142 = x_263; +x_143 = x_264; +x_144 = x_275; +x_145 = x_269; +x_146 = x_268; +x_147 = x_270; x_148 = x_295; x_149 = lean_box(0); goto block_230; @@ -8868,13 +8868,13 @@ lean_dec(x_281); lean_dec(x_279); lean_dec(x_275); lean_dec_ref(x_270); -lean_dec(x_269); -lean_dec_ref(x_267); -lean_dec(x_266); +lean_dec_ref(x_269); +lean_dec(x_268); lean_dec(x_264); -lean_dec(x_263); +lean_dec_ref(x_263); +lean_dec(x_262); lean_dec(x_260); -lean_dec_ref(x_259); +lean_dec(x_259); lean_dec_ref(x_258); lean_dec(x_6); x_296 = !lean_is_exclusive(x_294); @@ -8904,21 +8904,21 @@ lean_dec_ref(x_10); x_299 = lean_ctor_get(x_255, 0); lean_inc(x_299); lean_dec_ref(x_255); -x_133 = x_258; -x_134 = x_275; +x_133 = x_292; +x_134 = x_258; x_135 = x_259; -x_136 = x_292; -x_137 = x_260; -x_138 = x_279; -x_139 = x_263; -x_140 = x_264; -x_141 = x_291; -x_142 = x_286; -x_143 = x_267; -x_144 = x_266; -x_145 = x_270; -x_146 = x_269; -x_147 = x_281; +x_136 = x_291; +x_137 = x_279; +x_138 = x_281; +x_139 = x_286; +x_140 = x_260; +x_141 = x_262; +x_142 = x_263; +x_143 = x_264; +x_144 = x_275; +x_145 = x_269; +x_146 = x_268; +x_147 = x_270; x_148 = x_299; x_149 = lean_box(0); goto block_230; @@ -8932,17 +8932,17 @@ lean_dec(x_277); lean_dec(x_275); lean_dec(x_271); lean_dec_ref(x_270); -lean_dec(x_269); +lean_dec_ref(x_269); lean_dec(x_268); -lean_dec_ref(x_267); +lean_dec(x_267); lean_dec(x_266); lean_dec(x_265); lean_dec(x_264); -lean_dec(x_263); +lean_dec_ref(x_263); lean_dec(x_262); lean_dec(x_261); lean_dec(x_260); -lean_dec_ref(x_259); +lean_dec(x_259); lean_dec_ref(x_258); lean_dec(x_257); lean_dec_ref(x_231); @@ -8975,17 +8975,17 @@ lean_dec(x_277); lean_dec(x_275); lean_dec(x_271); lean_dec_ref(x_270); -lean_dec(x_269); +lean_dec_ref(x_269); lean_dec(x_268); -lean_dec_ref(x_267); +lean_dec(x_267); lean_dec(x_266); lean_dec(x_265); lean_dec(x_264); -lean_dec(x_263); +lean_dec_ref(x_263); lean_dec(x_262); lean_dec(x_261); lean_dec(x_260); -lean_dec_ref(x_259); +lean_dec(x_259); lean_dec_ref(x_258); lean_dec(x_257); lean_dec_ref(x_231); @@ -9017,17 +9017,17 @@ uint8_t x_306; lean_dec(x_275); lean_dec(x_271); lean_dec_ref(x_270); -lean_dec(x_269); +lean_dec_ref(x_269); lean_dec(x_268); -lean_dec_ref(x_267); +lean_dec(x_267); lean_dec(x_266); lean_dec(x_265); lean_dec(x_264); -lean_dec(x_263); +lean_dec_ref(x_263); lean_dec(x_262); lean_dec(x_261); lean_dec(x_260); -lean_dec_ref(x_259); +lean_dec(x_259); lean_dec_ref(x_258); lean_dec(x_257); lean_dec_ref(x_231); @@ -9057,17 +9057,17 @@ else { lean_dec(x_271); lean_dec_ref(x_270); -lean_dec(x_269); +lean_dec_ref(x_269); lean_dec(x_268); -lean_dec_ref(x_267); +lean_dec(x_267); lean_dec(x_266); lean_dec(x_265); lean_dec(x_264); -lean_dec(x_263); +lean_dec_ref(x_263); lean_dec(x_262); lean_dec(x_261); lean_dec(x_260); -lean_dec_ref(x_259); +lean_dec(x_259); lean_dec_ref(x_258); lean_dec(x_257); lean_dec_ref(x_231); @@ -9101,28 +9101,28 @@ x_325 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_326 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_327 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_328 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_313); +lean_inc(x_310); x_329 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_329, 0, x_313); +lean_ctor_set(x_329, 0, x_310); lean_ctor_set(x_329, 1, x_327); lean_ctor_set(x_329, 2, x_328); lean_inc_ref(x_329); -lean_inc(x_313); -x_330 = l_Lean_Syntax_node1(x_313, x_326, x_329); +lean_inc(x_310); +x_330 = l_Lean_Syntax_node1(x_310, x_326, x_329); x_331 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_332 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_333 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_334 = l_Lean_addMacroScope(x_317, x_333, x_311); -lean_inc(x_315); +x_334 = l_Lean_addMacroScope(x_317, x_333, x_316); lean_inc(x_313); +lean_inc(x_310); x_335 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_335, 0, x_313); +lean_ctor_set(x_335, 0, x_310); lean_ctor_set(x_335, 1, x_332); lean_ctor_set(x_335, 2, x_334); -lean_ctor_set(x_335, 3, x_315); -lean_inc(x_313); -x_336 = l_Lean_Syntax_node2(x_313, x_331, x_335, x_329); -x_337 = l_Lean_Syntax_node2(x_313, x_325, x_330, x_336); +lean_ctor_set(x_335, 3, x_313); +lean_inc(x_310); +x_336 = l_Lean_Syntax_node2(x_310, x_331, x_335, x_329); +x_337 = l_Lean_Syntax_node2(x_310, x_325, x_330, x_336); if (lean_obj_tag(x_255) == 0) { lean_object* x_338; lean_object* x_339; @@ -9134,21 +9134,21 @@ x_339 = lean_apply_3(x_338, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_339) == 0) { lean_dec_ref(x_339); -x_257 = x_320; -x_258 = x_322; -x_259 = x_323; -x_260 = x_327; -x_261 = x_331; -x_262 = x_325; -x_263 = x_316; -x_264 = x_310; +x_257 = x_312; +x_258 = x_324; +x_259 = x_313; +x_260 = x_315; +x_261 = x_320; +x_262 = x_311; +x_263 = x_323; +x_264 = x_327; x_265 = x_326; -x_266 = x_312; -x_267 = x_324; +x_266 = x_337; +x_267 = x_325; x_268 = x_314; -x_269 = x_315; -x_270 = x_328; -x_271 = x_337; +x_269 = x_328; +x_270 = x_322; +x_271 = x_331; x_272 = lean_box(0); goto block_309; } @@ -9157,11 +9157,11 @@ else uint8_t x_340; lean_dec(x_337); lean_dec(x_320); -lean_dec(x_316); lean_dec(x_315); lean_dec(x_314); +lean_dec(x_313); lean_dec(x_312); -lean_dec(x_310); +lean_dec(x_311); lean_dec_ref(x_231); lean_dec(x_11); lean_dec_ref(x_10); @@ -9188,21 +9188,21 @@ return x_342; } else { -x_257 = x_320; -x_258 = x_322; -x_259 = x_323; -x_260 = x_327; -x_261 = x_331; -x_262 = x_325; -x_263 = x_316; -x_264 = x_310; +x_257 = x_312; +x_258 = x_324; +x_259 = x_313; +x_260 = x_315; +x_261 = x_320; +x_262 = x_311; +x_263 = x_323; +x_264 = x_327; x_265 = x_326; -x_266 = x_312; -x_267 = x_324; +x_266 = x_337; +x_267 = x_325; x_268 = x_314; -x_269 = x_315; -x_270 = x_328; -x_271 = x_337; +x_269 = x_328; +x_270 = x_322; +x_271 = x_331; x_272 = lean_box(0); goto block_309; } @@ -9353,13 +9353,13 @@ lean_object* x_375; x_375 = lean_ctor_get(x_374, 0); lean_inc(x_375); lean_dec_ref(x_374); -x_310 = x_359; -x_311 = x_372; -x_312 = x_354; -x_313 = x_370; -x_314 = x_368; -x_315 = x_358; -x_316 = x_361; +x_310 = x_370; +x_311 = x_361; +x_312 = x_368; +x_313 = x_358; +x_314 = x_354; +x_315 = x_359; +x_316 = x_372; x_317 = x_375; x_318 = lean_box(0); goto block_349; @@ -9405,13 +9405,13 @@ lean_inc(x_379); lean_dec_ref(x_371); x_380 = lean_ctor_get(x_255, 0); lean_inc(x_380); -x_310 = x_359; -x_311 = x_379; -x_312 = x_354; -x_313 = x_370; -x_314 = x_368; -x_315 = x_358; -x_316 = x_361; +x_310 = x_370; +x_311 = x_361; +x_312 = x_368; +x_313 = x_358; +x_314 = x_354; +x_315 = x_359; +x_316 = x_379; x_317 = x_380; x_318 = lean_box(0); goto block_349; @@ -9760,22 +9760,22 @@ lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; x_449 = lean_ctor_get(x_448, 0); lean_inc(x_449); lean_dec_ref(x_448); -lean_inc_ref(x_438); -lean_inc(x_428); -lean_inc(x_425); +lean_inc_ref(x_437); +lean_inc(x_432); +lean_inc(x_429); x_450 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_450, 0, x_425); -lean_ctor_set(x_450, 1, x_428); -lean_ctor_set(x_450, 2, x_438); +lean_ctor_set(x_450, 0, x_429); +lean_ctor_set(x_450, 1, x_432); +lean_ctor_set(x_450, 2, x_437); lean_inc_ref(x_450); -lean_inc(x_425); -x_451 = l_Lean_Syntax_node1(x_425, x_433, x_450); -lean_inc(x_425); -x_452 = l_Lean_Syntax_node2(x_425, x_429, x_436, x_450); -x_453 = l_Lean_Syntax_node2(x_425, x_430, x_451, x_452); +lean_inc(x_429); +x_451 = l_Lean_Syntax_node1(x_429, x_433, x_450); +lean_inc(x_429); +x_452 = l_Lean_Syntax_node2(x_429, x_439, x_425, x_450); +x_453 = l_Lean_Syntax_node2(x_429, x_435, x_451, x_452); x_454 = lean_unsigned_to_nat(2u); x_455 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_456 = lean_array_push(x_455, x_439); +x_456 = lean_array_push(x_455, x_434); x_457 = lean_array_push(x_456, x_453); x_458 = l_Lake_DSL_expandAttrs(x_7); x_459 = l_Array_append___redArg(x_457, x_458); @@ -9792,21 +9792,21 @@ lean_object* x_463; x_463 = lean_ctor_get(x_462, 0); lean_inc(x_463); lean_dec_ref(x_462); -x_133 = x_426; -x_134 = x_443; +x_133 = x_460; +x_134 = x_426; x_135 = x_427; -x_136 = x_460; -x_137 = x_428; -x_138 = x_447; -x_139 = x_431; -x_140 = x_432; -x_141 = x_459; -x_142 = x_454; -x_143 = x_435; -x_144 = x_434; -x_145 = x_438; -x_146 = x_437; -x_147 = x_449; +x_136 = x_459; +x_137 = x_447; +x_138 = x_449; +x_139 = x_454; +x_140 = x_428; +x_141 = x_430; +x_142 = x_431; +x_143 = x_432; +x_144 = x_443; +x_145 = x_437; +x_146 = x_436; +x_147 = x_438; x_148 = x_463; x_149 = lean_box(0); goto block_230; @@ -9820,13 +9820,13 @@ lean_dec(x_449); lean_dec(x_447); lean_dec(x_443); lean_dec_ref(x_438); -lean_dec(x_437); -lean_dec_ref(x_435); -lean_dec(x_434); +lean_dec_ref(x_437); +lean_dec(x_436); lean_dec(x_432); -lean_dec(x_431); +lean_dec_ref(x_431); +lean_dec(x_430); lean_dec(x_428); -lean_dec_ref(x_427); +lean_dec(x_427); lean_dec_ref(x_426); lean_dec(x_6); x_464 = lean_ctor_get(x_462, 0); @@ -9857,21 +9857,21 @@ lean_dec_ref(x_10); x_467 = lean_ctor_get(x_423, 0); lean_inc(x_467); lean_dec_ref(x_423); -x_133 = x_426; -x_134 = x_443; +x_133 = x_460; +x_134 = x_426; x_135 = x_427; -x_136 = x_460; -x_137 = x_428; -x_138 = x_447; -x_139 = x_431; -x_140 = x_432; -x_141 = x_459; -x_142 = x_454; -x_143 = x_435; -x_144 = x_434; -x_145 = x_438; -x_146 = x_437; -x_147 = x_449; +x_136 = x_459; +x_137 = x_447; +x_138 = x_449; +x_139 = x_454; +x_140 = x_428; +x_141 = x_430; +x_142 = x_431; +x_143 = x_432; +x_144 = x_443; +x_145 = x_437; +x_146 = x_436; +x_147 = x_438; x_148 = x_467; x_149 = lean_box(0); goto block_230; @@ -9885,17 +9885,17 @@ lean_dec(x_445); lean_dec(x_443); lean_dec(x_439); lean_dec_ref(x_438); -lean_dec(x_437); +lean_dec_ref(x_437); lean_dec(x_436); -lean_dec_ref(x_435); +lean_dec(x_435); lean_dec(x_434); lean_dec(x_433); lean_dec(x_432); -lean_dec(x_431); +lean_dec_ref(x_431); lean_dec(x_430); lean_dec(x_429); lean_dec(x_428); -lean_dec_ref(x_427); +lean_dec(x_427); lean_dec_ref(x_426); lean_dec(x_425); lean_dec_ref(x_231); @@ -9929,17 +9929,17 @@ lean_dec(x_445); lean_dec(x_443); lean_dec(x_439); lean_dec_ref(x_438); -lean_dec(x_437); +lean_dec_ref(x_437); lean_dec(x_436); -lean_dec_ref(x_435); +lean_dec(x_435); lean_dec(x_434); lean_dec(x_433); lean_dec(x_432); -lean_dec(x_431); +lean_dec_ref(x_431); lean_dec(x_430); lean_dec(x_429); lean_dec(x_428); -lean_dec_ref(x_427); +lean_dec(x_427); lean_dec_ref(x_426); lean_dec(x_425); lean_dec_ref(x_231); @@ -9972,17 +9972,17 @@ lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_dec(x_443); lean_dec(x_439); lean_dec_ref(x_438); -lean_dec(x_437); +lean_dec_ref(x_437); lean_dec(x_436); -lean_dec_ref(x_435); +lean_dec(x_435); lean_dec(x_434); lean_dec(x_433); lean_dec(x_432); -lean_dec(x_431); +lean_dec_ref(x_431); lean_dec(x_430); lean_dec(x_429); lean_dec(x_428); -lean_dec_ref(x_427); +lean_dec(x_427); lean_dec_ref(x_426); lean_dec(x_425); lean_dec_ref(x_231); @@ -10013,17 +10013,17 @@ else { lean_dec(x_439); lean_dec_ref(x_438); -lean_dec(x_437); +lean_dec_ref(x_437); lean_dec(x_436); -lean_dec_ref(x_435); +lean_dec(x_435); lean_dec(x_434); lean_dec(x_433); lean_dec(x_432); -lean_dec(x_431); +lean_dec_ref(x_431); lean_dec(x_430); lean_dec(x_429); lean_dec(x_428); -lean_dec_ref(x_427); +lean_dec(x_427); lean_dec_ref(x_426); lean_dec(x_425); lean_dec_ref(x_231); @@ -10057,28 +10057,28 @@ x_493 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_494 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_495 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_496 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_481); +lean_inc(x_478); x_497 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_497, 0, x_481); +lean_ctor_set(x_497, 0, x_478); lean_ctor_set(x_497, 1, x_495); lean_ctor_set(x_497, 2, x_496); lean_inc_ref(x_497); -lean_inc(x_481); -x_498 = l_Lean_Syntax_node1(x_481, x_494, x_497); +lean_inc(x_478); +x_498 = l_Lean_Syntax_node1(x_478, x_494, x_497); x_499 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_500 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_501 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_502 = l_Lean_addMacroScope(x_485, x_501, x_479); -lean_inc(x_483); +x_502 = l_Lean_addMacroScope(x_485, x_501, x_484); lean_inc(x_481); +lean_inc(x_478); x_503 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_503, 0, x_481); +lean_ctor_set(x_503, 0, x_478); lean_ctor_set(x_503, 1, x_500); lean_ctor_set(x_503, 2, x_502); -lean_ctor_set(x_503, 3, x_483); -lean_inc(x_481); -x_504 = l_Lean_Syntax_node2(x_481, x_499, x_503, x_497); -x_505 = l_Lean_Syntax_node2(x_481, x_493, x_498, x_504); +lean_ctor_set(x_503, 3, x_481); +lean_inc(x_478); +x_504 = l_Lean_Syntax_node2(x_478, x_499, x_503, x_497); +x_505 = l_Lean_Syntax_node2(x_478, x_493, x_498, x_504); if (lean_obj_tag(x_423) == 0) { lean_object* x_506; lean_object* x_507; @@ -10090,21 +10090,21 @@ x_507 = lean_apply_3(x_506, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_507) == 0) { lean_dec_ref(x_507); -x_425 = x_488; -x_426 = x_490; -x_427 = x_491; -x_428 = x_495; -x_429 = x_499; -x_430 = x_493; -x_431 = x_484; -x_432 = x_478; +x_425 = x_480; +x_426 = x_492; +x_427 = x_481; +x_428 = x_483; +x_429 = x_488; +x_430 = x_479; +x_431 = x_491; +x_432 = x_495; x_433 = x_494; -x_434 = x_480; -x_435 = x_492; +x_434 = x_505; +x_435 = x_493; x_436 = x_482; -x_437 = x_483; -x_438 = x_496; -x_439 = x_505; +x_437 = x_496; +x_438 = x_490; +x_439 = x_499; x_440 = lean_box(0); goto block_477; } @@ -10113,11 +10113,11 @@ else lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_dec(x_505); lean_dec(x_488); -lean_dec(x_484); lean_dec(x_483); lean_dec(x_482); +lean_dec(x_481); lean_dec(x_480); -lean_dec(x_478); +lean_dec(x_479); lean_dec_ref(x_231); lean_dec(x_11); lean_dec_ref(x_10); @@ -10145,21 +10145,21 @@ return x_510; } else { -x_425 = x_488; -x_426 = x_490; -x_427 = x_491; -x_428 = x_495; -x_429 = x_499; -x_430 = x_493; -x_431 = x_484; -x_432 = x_478; +x_425 = x_480; +x_426 = x_492; +x_427 = x_481; +x_428 = x_483; +x_429 = x_488; +x_430 = x_479; +x_431 = x_491; +x_432 = x_495; x_433 = x_494; -x_434 = x_480; -x_435 = x_492; +x_434 = x_505; +x_435 = x_493; x_436 = x_482; -x_437 = x_483; -x_438 = x_496; -x_439 = x_505; +x_437 = x_496; +x_438 = x_490; +x_439 = x_499; x_440 = lean_box(0); goto block_477; } @@ -10312,13 +10312,13 @@ lean_object* x_543; x_543 = lean_ctor_get(x_542, 0); lean_inc(x_543); lean_dec_ref(x_542); -x_478 = x_527; -x_479 = x_540; -x_480 = x_522; -x_481 = x_538; -x_482 = x_536; -x_483 = x_526; -x_484 = x_529; +x_478 = x_538; +x_479 = x_529; +x_480 = x_536; +x_481 = x_526; +x_482 = x_522; +x_483 = x_527; +x_484 = x_540; x_485 = x_543; x_486 = lean_box(0); goto block_517; @@ -10365,13 +10365,13 @@ lean_inc(x_547); lean_dec_ref(x_539); x_548 = lean_ctor_get(x_423, 0); lean_inc(x_548); -x_478 = x_527; -x_479 = x_547; -x_480 = x_522; -x_481 = x_538; -x_482 = x_536; -x_483 = x_526; -x_484 = x_529; +x_478 = x_538; +x_479 = x_529; +x_480 = x_536; +x_481 = x_526; +x_482 = x_522; +x_483 = x_527; +x_484 = x_547; x_485 = x_548; x_486 = lean_box(0); goto block_517; @@ -10744,22 +10744,22 @@ lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; x_620 = lean_ctor_get(x_619, 0); lean_inc(x_620); lean_dec_ref(x_619); -lean_inc_ref(x_609); -lean_inc(x_599); -lean_inc(x_596); +lean_inc_ref(x_608); +lean_inc(x_603); +lean_inc(x_600); x_621 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_621, 0, x_596); -lean_ctor_set(x_621, 1, x_599); -lean_ctor_set(x_621, 2, x_609); +lean_ctor_set(x_621, 0, x_600); +lean_ctor_set(x_621, 1, x_603); +lean_ctor_set(x_621, 2, x_608); lean_inc_ref(x_621); -lean_inc(x_596); -x_622 = l_Lean_Syntax_node1(x_596, x_604, x_621); -lean_inc(x_596); -x_623 = l_Lean_Syntax_node2(x_596, x_600, x_607, x_621); -x_624 = l_Lean_Syntax_node2(x_596, x_601, x_622, x_623); +lean_inc(x_600); +x_622 = l_Lean_Syntax_node1(x_600, x_604, x_621); +lean_inc(x_600); +x_623 = l_Lean_Syntax_node2(x_600, x_610, x_596, x_621); +x_624 = l_Lean_Syntax_node2(x_600, x_606, x_622, x_623); x_625 = lean_unsigned_to_nat(2u); x_626 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_627 = lean_array_push(x_626, x_610); +x_627 = lean_array_push(x_626, x_605); x_628 = lean_array_push(x_627, x_624); x_629 = l_Lake_DSL_expandAttrs(x_7); x_630 = l_Array_append___redArg(x_628, x_629); @@ -10776,21 +10776,21 @@ lean_object* x_634; x_634 = lean_ctor_get(x_633, 0); lean_inc(x_634); lean_dec_ref(x_633); -x_133 = x_597; -x_134 = x_614; +x_133 = x_631; +x_134 = x_597; x_135 = x_598; -x_136 = x_631; -x_137 = x_599; -x_138 = x_618; -x_139 = x_602; -x_140 = x_603; -x_141 = x_630; -x_142 = x_625; -x_143 = x_606; -x_144 = x_605; -x_145 = x_609; -x_146 = x_608; -x_147 = x_620; +x_136 = x_630; +x_137 = x_618; +x_138 = x_620; +x_139 = x_625; +x_140 = x_599; +x_141 = x_601; +x_142 = x_602; +x_143 = x_603; +x_144 = x_614; +x_145 = x_608; +x_146 = x_607; +x_147 = x_609; x_148 = x_634; x_149 = lean_box(0); goto block_230; @@ -10804,13 +10804,13 @@ lean_dec(x_620); lean_dec(x_618); lean_dec(x_614); lean_dec_ref(x_609); -lean_dec(x_608); -lean_dec_ref(x_606); -lean_dec(x_605); +lean_dec_ref(x_608); +lean_dec(x_607); lean_dec(x_603); -lean_dec(x_602); +lean_dec_ref(x_602); +lean_dec(x_601); lean_dec(x_599); -lean_dec_ref(x_598); +lean_dec(x_598); lean_dec_ref(x_597); lean_dec(x_6); x_635 = lean_ctor_get(x_633, 0); @@ -10841,21 +10841,21 @@ lean_dec_ref(x_10); x_638 = lean_ctor_get(x_594, 0); lean_inc(x_638); lean_dec_ref(x_594); -x_133 = x_597; -x_134 = x_614; +x_133 = x_631; +x_134 = x_597; x_135 = x_598; -x_136 = x_631; -x_137 = x_599; -x_138 = x_618; -x_139 = x_602; -x_140 = x_603; -x_141 = x_630; -x_142 = x_625; -x_143 = x_606; -x_144 = x_605; -x_145 = x_609; -x_146 = x_608; -x_147 = x_620; +x_136 = x_630; +x_137 = x_618; +x_138 = x_620; +x_139 = x_625; +x_140 = x_599; +x_141 = x_601; +x_142 = x_602; +x_143 = x_603; +x_144 = x_614; +x_145 = x_608; +x_146 = x_607; +x_147 = x_609; x_148 = x_638; x_149 = lean_box(0); goto block_230; @@ -10869,17 +10869,17 @@ lean_dec(x_616); lean_dec(x_614); lean_dec(x_610); lean_dec_ref(x_609); -lean_dec(x_608); +lean_dec_ref(x_608); lean_dec(x_607); -lean_dec_ref(x_606); +lean_dec(x_606); lean_dec(x_605); lean_dec(x_604); lean_dec(x_603); -lean_dec(x_602); +lean_dec_ref(x_602); lean_dec(x_601); lean_dec(x_600); lean_dec(x_599); -lean_dec_ref(x_598); +lean_dec(x_598); lean_dec_ref(x_597); lean_dec(x_596); lean_dec_ref(x_587); @@ -10913,17 +10913,17 @@ lean_dec(x_616); lean_dec(x_614); lean_dec(x_610); lean_dec_ref(x_609); -lean_dec(x_608); +lean_dec_ref(x_608); lean_dec(x_607); -lean_dec_ref(x_606); +lean_dec(x_606); lean_dec(x_605); lean_dec(x_604); lean_dec(x_603); -lean_dec(x_602); +lean_dec_ref(x_602); lean_dec(x_601); lean_dec(x_600); lean_dec(x_599); -lean_dec_ref(x_598); +lean_dec(x_598); lean_dec_ref(x_597); lean_dec(x_596); lean_dec_ref(x_587); @@ -10956,17 +10956,17 @@ lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_dec(x_614); lean_dec(x_610); lean_dec_ref(x_609); -lean_dec(x_608); +lean_dec_ref(x_608); lean_dec(x_607); -lean_dec_ref(x_606); +lean_dec(x_606); lean_dec(x_605); lean_dec(x_604); lean_dec(x_603); -lean_dec(x_602); +lean_dec_ref(x_602); lean_dec(x_601); lean_dec(x_600); lean_dec(x_599); -lean_dec_ref(x_598); +lean_dec(x_598); lean_dec_ref(x_597); lean_dec(x_596); lean_dec_ref(x_587); @@ -10997,17 +10997,17 @@ else { lean_dec(x_610); lean_dec_ref(x_609); -lean_dec(x_608); +lean_dec_ref(x_608); lean_dec(x_607); -lean_dec_ref(x_606); +lean_dec(x_606); lean_dec(x_605); lean_dec(x_604); lean_dec(x_603); -lean_dec(x_602); +lean_dec_ref(x_602); lean_dec(x_601); lean_dec(x_600); lean_dec(x_599); -lean_dec_ref(x_598); +lean_dec(x_598); lean_dec_ref(x_597); lean_dec(x_596); lean_dec_ref(x_587); @@ -11041,28 +11041,28 @@ x_664 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_665 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_666 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_667 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_652); +lean_inc(x_649); x_668 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_668, 0, x_652); +lean_ctor_set(x_668, 0, x_649); lean_ctor_set(x_668, 1, x_666); lean_ctor_set(x_668, 2, x_667); lean_inc_ref(x_668); -lean_inc(x_652); -x_669 = l_Lean_Syntax_node1(x_652, x_665, x_668); +lean_inc(x_649); +x_669 = l_Lean_Syntax_node1(x_649, x_665, x_668); x_670 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_671 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_672 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_673 = l_Lean_addMacroScope(x_656, x_672, x_650); -lean_inc(x_654); +x_673 = l_Lean_addMacroScope(x_656, x_672, x_655); lean_inc(x_652); +lean_inc(x_649); x_674 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_674, 0, x_652); +lean_ctor_set(x_674, 0, x_649); lean_ctor_set(x_674, 1, x_671); lean_ctor_set(x_674, 2, x_673); -lean_ctor_set(x_674, 3, x_654); -lean_inc(x_652); -x_675 = l_Lean_Syntax_node2(x_652, x_670, x_674, x_668); -x_676 = l_Lean_Syntax_node2(x_652, x_664, x_669, x_675); +lean_ctor_set(x_674, 3, x_652); +lean_inc(x_649); +x_675 = l_Lean_Syntax_node2(x_649, x_670, x_674, x_668); +x_676 = l_Lean_Syntax_node2(x_649, x_664, x_669, x_675); if (lean_obj_tag(x_594) == 0) { lean_object* x_677; lean_object* x_678; @@ -11074,21 +11074,21 @@ x_678 = lean_apply_3(x_677, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_678) == 0) { lean_dec_ref(x_678); -x_596 = x_659; -x_597 = x_661; -x_598 = x_662; -x_599 = x_666; -x_600 = x_670; -x_601 = x_664; -x_602 = x_655; -x_603 = x_649; +x_596 = x_651; +x_597 = x_663; +x_598 = x_652; +x_599 = x_654; +x_600 = x_659; +x_601 = x_650; +x_602 = x_662; +x_603 = x_666; x_604 = x_665; -x_605 = x_651; -x_606 = x_663; +x_605 = x_676; +x_606 = x_664; x_607 = x_653; -x_608 = x_654; -x_609 = x_667; -x_610 = x_676; +x_608 = x_667; +x_609 = x_661; +x_610 = x_670; x_611 = lean_box(0); goto block_648; } @@ -11097,11 +11097,11 @@ else lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_dec(x_676); lean_dec(x_659); -lean_dec(x_655); lean_dec(x_654); lean_dec(x_653); +lean_dec(x_652); lean_dec(x_651); -lean_dec(x_649); +lean_dec(x_650); lean_dec_ref(x_587); lean_dec(x_11); lean_dec_ref(x_10); @@ -11129,21 +11129,21 @@ return x_681; } else { -x_596 = x_659; -x_597 = x_661; -x_598 = x_662; -x_599 = x_666; -x_600 = x_670; -x_601 = x_664; -x_602 = x_655; -x_603 = x_649; +x_596 = x_651; +x_597 = x_663; +x_598 = x_652; +x_599 = x_654; +x_600 = x_659; +x_601 = x_650; +x_602 = x_662; +x_603 = x_666; x_604 = x_665; -x_605 = x_651; -x_606 = x_663; +x_605 = x_676; +x_606 = x_664; x_607 = x_653; -x_608 = x_654; -x_609 = x_667; -x_610 = x_676; +x_608 = x_667; +x_609 = x_661; +x_610 = x_670; x_611 = lean_box(0); goto block_648; } @@ -11296,13 +11296,13 @@ lean_object* x_714; x_714 = lean_ctor_get(x_713, 0); lean_inc(x_714); lean_dec_ref(x_713); -x_649 = x_698; -x_650 = x_711; -x_651 = x_693; -x_652 = x_709; -x_653 = x_707; -x_654 = x_697; -x_655 = x_700; +x_649 = x_709; +x_650 = x_700; +x_651 = x_707; +x_652 = x_697; +x_653 = x_693; +x_654 = x_698; +x_655 = x_711; x_656 = x_714; x_657 = lean_box(0); goto block_688; @@ -11349,13 +11349,13 @@ lean_inc(x_718); lean_dec_ref(x_710); x_719 = lean_ctor_get(x_594, 0); lean_inc(x_719); -x_649 = x_698; -x_650 = x_718; -x_651 = x_693; -x_652 = x_709; -x_653 = x_707; -x_654 = x_697; -x_655 = x_700; +x_649 = x_709; +x_650 = x_700; +x_651 = x_707; +x_652 = x_697; +x_653 = x_693; +x_654 = x_698; +x_655 = x_718; x_656 = x_719; x_657 = lean_box(0); goto block_688; @@ -11560,43 +11560,43 @@ return x_742; block_132: { 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_inc_ref(x_26); -x_44 = l_Array_append___redArg(x_26, x_43); +lean_inc_ref(x_41); +x_44 = l_Array_append___redArg(x_41, x_43); lean_dec_ref(x_43); -lean_inc(x_32); -lean_inc(x_33); +lean_inc(x_26); +lean_inc(x_19); x_45 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_45, 0, x_33); -lean_ctor_set(x_45, 1, x_32); +lean_ctor_set(x_45, 0, x_19); +lean_ctor_set(x_45, 1, x_26); lean_ctor_set(x_45, 2, x_44); -lean_inc_n(x_41, 6); -lean_inc(x_13); -lean_inc(x_33); -x_46 = l_Lean_Syntax_node7(x_33, x_13, x_45, x_41, x_41, x_41, x_41, x_41, x_41); +lean_inc_n(x_14, 6); +lean_inc(x_21); +lean_inc(x_19); +x_46 = l_Lean_Syntax_node7(x_19, x_21, x_45, x_14, x_14, x_14, x_14, x_14, x_14); x_47 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_14); +lean_inc_ref(x_22); +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_48 = l_Lean_Name_mkStr4(x_16, x_31, x_14, x_47); -lean_inc(x_33); +x_48 = l_Lean_Name_mkStr4(x_31, x_24, x_22, x_47); +lean_inc(x_19); x_49 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_49, 0, x_33); +lean_ctor_set(x_49, 0, x_19); lean_ctor_set(x_49, 1, x_47); x_50 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_14); +lean_inc_ref(x_22); +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_51 = l_Lean_Name_mkStr4(x_16, x_31, x_14, x_50); +x_51 = l_Lean_Name_mkStr4(x_31, x_24, x_22, x_50); x_52 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_53 = lean_box(2); -lean_inc(x_32); +lean_inc(x_26); x_54 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_32); +lean_ctor_set(x_54, 1, x_26); lean_ctor_set(x_54, 2, x_52); -x_55 = lean_mk_empty_array_with_capacity(x_24); -lean_inc(x_37); -x_56 = lean_array_push(x_55, x_37); +x_55 = lean_mk_empty_array_with_capacity(x_18); +lean_inc(x_28); +x_56 = lean_array_push(x_55, x_28); x_57 = lean_array_push(x_56, x_54); lean_inc(x_51); x_58 = lean_alloc_ctor(1, 3, 0); @@ -11604,194 +11604,194 @@ lean_ctor_set(x_58, 0, x_53); lean_ctor_set(x_58, 1, x_51); lean_ctor_set(x_58, 2, x_57); x_59 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_14); +lean_inc_ref(x_22); +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_60 = l_Lean_Name_mkStr4(x_16, x_31, x_14, x_59); +x_60 = l_Lean_Name_mkStr4(x_31, x_24, x_22, x_59); x_61 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_25); -lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_62 = l_Lean_Name_mkStr4(x_16, x_31, x_25, x_61); -lean_inc(x_29); +lean_inc_ref(x_15); +lean_inc_ref(x_24); +lean_inc_ref(x_31); +x_62 = l_Lean_Name_mkStr4(x_31, x_24, x_15, x_61); +lean_inc(x_30); lean_inc(x_62); -lean_inc(x_33); -x_63 = l_Lean_Syntax_node2(x_33, x_62, x_29, x_30); -lean_inc(x_32); -lean_inc(x_33); -x_64 = l_Lean_Syntax_node1(x_33, x_32, x_63); -lean_inc(x_41); +lean_inc(x_19); +x_63 = l_Lean_Syntax_node2(x_19, x_62, x_30, x_27); +lean_inc(x_26); +lean_inc(x_19); +x_64 = l_Lean_Syntax_node1(x_19, x_26, x_63); +lean_inc(x_14); lean_inc(x_60); -lean_inc(x_33); -x_65 = l_Lean_Syntax_node2(x_33, x_60, x_41, x_64); +lean_inc(x_19); +x_65 = l_Lean_Syntax_node2(x_19, x_60, x_14, x_64); x_66 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__60; -lean_inc_ref(x_14); +lean_inc_ref(x_22); +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_67 = l_Lean_Name_mkStr4(x_16, x_31, x_14, x_66); +x_67 = l_Lean_Name_mkStr4(x_31, x_24, x_22, x_66); x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__1; x_69 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__2; -lean_inc_ref(x_23); -x_70 = l_Lean_Name_mkStr3(x_23, x_15, x_69); -lean_inc(x_42); +lean_inc_ref(x_34); +x_70 = l_Lean_Name_mkStr3(x_34, x_32, x_69); +lean_inc(x_37); lean_inc(x_70); -lean_inc(x_17); -x_71 = l_Lean_addMacroScope(x_17, x_70, x_42); -lean_inc(x_28); +lean_inc(x_23); +x_71 = l_Lean_addMacroScope(x_23, x_70, x_37); +lean_inc(x_33); x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_28); -lean_inc(x_27); +lean_ctor_set(x_72, 1, x_33); +lean_inc(x_17); x_73 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_27); -lean_inc(x_33); +lean_ctor_set(x_73, 1, x_17); +lean_inc(x_19); x_74 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_74, 0, x_33); +lean_ctor_set(x_74, 0, x_19); lean_ctor_set(x_74, 1, x_68); lean_ctor_set(x_74, 2, x_71); lean_ctor_set(x_74, 3, x_73); -lean_inc(x_32); -lean_inc(x_33); -x_75 = l_Lean_Syntax_node4(x_33, x_32, x_36, x_34, x_18, x_21); -lean_inc(x_33); -x_76 = l_Lean_Syntax_node2(x_33, x_40, x_74, x_75); +lean_inc(x_26); +lean_inc(x_19); +x_75 = l_Lean_Syntax_node4(x_19, x_26, x_29, x_39, x_13, x_38); +lean_inc(x_19); +x_76 = l_Lean_Syntax_node2(x_19, x_42, x_74, x_75); x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__62; x_78 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__63; +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_79 = l_Lean_Name_mkStr4(x_16, x_31, x_77, x_78); -lean_inc_n(x_41, 2); -lean_inc(x_33); -x_80 = l_Lean_Syntax_node2(x_33, x_79, x_41, x_41); -lean_inc(x_41); +x_79 = l_Lean_Name_mkStr4(x_31, x_24, x_77, x_78); +lean_inc_n(x_14, 2); +lean_inc(x_19); +x_80 = l_Lean_Syntax_node2(x_19, x_79, x_14, x_14); +lean_inc(x_14); lean_inc(x_80); -lean_inc(x_38); +lean_inc(x_16); lean_inc(x_67); -lean_inc(x_33); -x_81 = l_Lean_Syntax_node4(x_33, x_67, x_38, x_76, x_80, x_41); -lean_inc(x_33); -x_82 = l_Lean_Syntax_node4(x_33, x_48, x_49, x_58, x_65, x_81); +lean_inc(x_19); +x_81 = l_Lean_Syntax_node4(x_19, x_67, x_16, x_76, x_80, x_14); +lean_inc(x_19); +x_82 = l_Lean_Syntax_node4(x_19, x_48, x_49, x_58, x_65, x_81); lean_inc(x_20); -lean_inc(x_33); -x_83 = l_Lean_Syntax_node2(x_33, x_20, x_46, x_82); +lean_inc(x_19); +x_83 = l_Lean_Syntax_node2(x_19, x_20, x_46, x_82); x_84 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_25); +lean_inc_ref(x_15); +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_85 = l_Lean_Name_mkStr4(x_16, x_31, x_25, x_84); +x_85 = l_Lean_Name_mkStr4(x_31, x_24, x_15, x_84); x_86 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_33); +lean_inc(x_19); x_87 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_87, 0, x_33); +lean_ctor_set(x_87, 0, x_19); lean_ctor_set(x_87, 1, x_86); -x_88 = l_Lean_Syntax_SepArray_ofElems(x_39, x_22); -lean_dec_ref(x_22); -x_89 = l_Array_append___redArg(x_26, x_88); +x_88 = l_Lean_Syntax_SepArray_ofElems(x_35, x_36); +lean_dec_ref(x_36); +x_89 = l_Array_append___redArg(x_41, x_88); lean_dec_ref(x_88); -lean_inc(x_32); -lean_inc(x_33); +lean_inc(x_26); +lean_inc(x_19); x_90 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_90, 0, x_33); -lean_ctor_set(x_90, 1, x_32); +lean_ctor_set(x_90, 0, x_19); +lean_ctor_set(x_90, 1, x_26); lean_ctor_set(x_90, 2, x_89); x_91 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_33); +lean_inc(x_19); x_92 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_92, 0, x_33); +lean_ctor_set(x_92, 0, x_19); lean_ctor_set(x_92, 1, x_91); -lean_inc(x_33); -x_93 = l_Lean_Syntax_node3(x_33, x_85, x_87, x_90, x_92); -lean_inc(x_32); -lean_inc(x_33); -x_94 = l_Lean_Syntax_node1(x_33, x_32, x_93); -lean_inc_n(x_41, 6); -lean_inc(x_33); -x_95 = l_Lean_Syntax_node7(x_33, x_13, x_41, x_94, x_41, x_41, x_41, x_41, x_41); +lean_inc(x_19); +x_93 = l_Lean_Syntax_node3(x_19, x_85, x_87, x_90, x_92); +lean_inc(x_26); +lean_inc(x_19); +x_94 = l_Lean_Syntax_node1(x_19, x_26, x_93); +lean_inc_n(x_14, 6); +lean_inc(x_19); +x_95 = l_Lean_Syntax_node7(x_19, x_21, x_14, x_94, x_14, x_14, x_14, x_14, x_14); x_96 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; +lean_inc_ref(x_24); lean_inc_ref(x_31); -lean_inc_ref(x_16); -x_97 = l_Lean_Name_mkStr4(x_16, x_31, x_14, x_96); +x_97 = l_Lean_Name_mkStr4(x_31, x_24, x_22, x_96); x_98 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_33); +lean_inc(x_19); x_99 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_99, 0, x_33); +lean_ctor_set(x_99, 0, x_19); lean_ctor_set(x_99, 1, x_98); x_100 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_101 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_42); +lean_inc(x_37); +lean_inc(x_23); +x_102 = l_Lean_addMacroScope(x_23, x_101, x_37); lean_inc(x_17); -x_102 = l_Lean_addMacroScope(x_17, x_101, x_42); -lean_inc(x_27); -lean_inc(x_33); +lean_inc(x_19); x_103 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_103, 0, x_33); +lean_ctor_set(x_103, 0, x_19); lean_ctor_set(x_103, 1, x_100); lean_ctor_set(x_103, 2, x_102); -lean_ctor_set(x_103, 3, x_27); -lean_inc(x_41); -lean_inc(x_33); -x_104 = l_Lean_Syntax_node2(x_33, x_51, x_103, x_41); +lean_ctor_set(x_103, 3, x_17); +lean_inc(x_14); +lean_inc(x_19); +x_104 = l_Lean_Syntax_node2(x_19, x_51, x_103, x_14); x_105 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__5; x_106 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_107 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_42); -lean_inc(x_17); -x_108 = l_Lean_addMacroScope(x_17, x_107, x_42); -x_109 = l_Lean_Name_mkStr2(x_23, x_105); +lean_inc(x_37); +lean_inc(x_23); +x_108 = l_Lean_addMacroScope(x_23, x_107, x_37); +x_109 = l_Lean_Name_mkStr2(x_34, x_105); lean_inc(x_109); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_28); +lean_ctor_set(x_110, 1, x_33); x_111 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_111, 0, x_109); -lean_inc(x_27); +lean_inc(x_17); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_111); -lean_ctor_set(x_112, 1, x_27); +lean_ctor_set(x_112, 1, x_17); x_113 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_113, 0, x_110); lean_ctor_set(x_113, 1, x_112); -lean_inc(x_33); +lean_inc(x_19); x_114 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_114, 0, x_33); +lean_ctor_set(x_114, 0, x_19); lean_ctor_set(x_114, 1, x_106); lean_ctor_set(x_114, 2, x_108); lean_ctor_set(x_114, 3, x_113); -lean_inc(x_33); -x_115 = l_Lean_Syntax_node2(x_33, x_62, x_29, x_114); -lean_inc(x_32); -lean_inc(x_33); -x_116 = l_Lean_Syntax_node1(x_33, x_32, x_115); -lean_inc(x_41); -lean_inc(x_33); -x_117 = l_Lean_Syntax_node2(x_33, x_60, x_41, x_116); +lean_inc(x_19); +x_115 = l_Lean_Syntax_node2(x_19, x_62, x_30, x_114); +lean_inc(x_26); +lean_inc(x_19); +x_116 = l_Lean_Syntax_node1(x_19, x_26, x_115); +lean_inc(x_14); +lean_inc(x_19); +x_117 = l_Lean_Syntax_node2(x_19, x_60, x_14, x_116); x_118 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_119 = l_Lean_Name_mkStr4(x_16, x_31, x_25, x_118); +x_119 = l_Lean_Name_mkStr4(x_31, x_24, x_15, x_118); x_120 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_33); +lean_inc(x_19); x_121 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_121, 0, x_33); +lean_ctor_set(x_121, 0, x_19); lean_ctor_set(x_121, 1, x_120); x_122 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_123 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_124 = l_Lean_addMacroScope(x_17, x_123, x_42); -lean_inc(x_33); +x_124 = l_Lean_addMacroScope(x_23, x_123, x_37); +lean_inc(x_19); x_125 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_125, 0, x_33); +lean_ctor_set(x_125, 0, x_19); lean_ctor_set(x_125, 1, x_122); lean_ctor_set(x_125, 2, x_124); -lean_ctor_set(x_125, 3, x_27); -lean_inc(x_33); -x_126 = l_Lean_Syntax_node3(x_33, x_119, x_37, x_121, x_125); -lean_inc(x_41); -lean_inc(x_33); -x_127 = l_Lean_Syntax_node4(x_33, x_67, x_38, x_126, x_80, x_41); -lean_inc(x_33); -x_128 = l_Lean_Syntax_node5(x_33, x_97, x_99, x_104, x_117, x_127, x_41); -lean_inc(x_33); -x_129 = l_Lean_Syntax_node2(x_33, x_20, x_95, x_128); -x_130 = l_Lean_Syntax_node3(x_33, x_32, x_19, x_83, x_129); +lean_ctor_set(x_125, 3, x_17); +lean_inc(x_19); +x_126 = l_Lean_Syntax_node3(x_19, x_119, x_28, x_121, x_125); +lean_inc(x_14); +lean_inc(x_19); +x_127 = l_Lean_Syntax_node4(x_19, x_67, x_16, x_126, x_80, x_14); +lean_inc(x_19); +x_128 = l_Lean_Syntax_node5(x_19, x_97, x_99, x_104, x_117, x_127, x_14); +lean_inc(x_19); +x_129 = l_Lean_Syntax_node2(x_19, x_20, x_95, x_128); +x_130 = l_Lean_Syntax_node3(x_19, x_26, x_25, x_83, x_129); x_131 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_131, 0, x_130); return x_131; @@ -11802,90 +11802,90 @@ lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__0; x_151 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; lean_inc_ref(x_145); +lean_inc(x_143); lean_inc(x_137); -lean_inc(x_138); x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_138); -lean_ctor_set(x_152, 1, x_137); +lean_ctor_set(x_152, 0, x_137); +lean_ctor_set(x_152, 1, x_143); lean_ctor_set(x_152, 2, x_145); x_153 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; -lean_inc(x_138); +lean_inc(x_137); x_154 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_154, 0, x_138); +lean_ctor_set(x_154, 0, x_137); lean_ctor_set(x_154, 1, x_153); x_155 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_138); +lean_inc(x_137); x_156 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_156, 0, x_138); +lean_ctor_set(x_156, 0, x_137); lean_ctor_set(x_156, 1, x_155); x_157 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__30; x_158 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__31; -lean_inc(x_147); +lean_inc(x_138); lean_inc(x_148); -x_159 = l_Lean_addMacroScope(x_148, x_158, x_147); +x_159 = l_Lean_addMacroScope(x_148, x_158, x_138); x_160 = lean_box(0); x_161 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__3; -lean_inc(x_146); +lean_inc(x_135); x_162 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_162, 0, x_161); -lean_ctor_set(x_162, 1, x_146); -lean_inc(x_138); +lean_ctor_set(x_162, 1, x_135); +lean_inc(x_137); x_163 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_163, 0, x_138); +lean_ctor_set(x_163, 0, x_137); lean_ctor_set(x_163, 1, x_157); lean_ctor_set(x_163, 2, x_159); lean_ctor_set(x_163, 3, x_162); x_164 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_143); -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_165 = l_Lean_Name_mkStr4(x_133, x_135, x_143, x_164); +lean_inc_ref(x_134); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_165 = l_Lean_Name_mkStr4(x_147, x_142, x_134, x_164); x_166 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_143); -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_167 = l_Lean_Name_mkStr4(x_133, x_135, x_143, x_166); +lean_inc_ref(x_134); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_167 = l_Lean_Name_mkStr4(x_147, x_142, x_134, x_166); x_168 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; -lean_inc(x_138); +lean_inc(x_137); x_169 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_169, 0, x_138); +lean_ctor_set(x_169, 0, x_137); lean_ctor_set(x_169, 1, x_168); x_170 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__25; x_171 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__27; x_172 = lean_box(0); -lean_inc(x_147); +lean_inc(x_138); lean_inc(x_148); -x_173 = l_Lean_addMacroScope(x_148, x_172, x_147); +x_173 = l_Lean_addMacroScope(x_148, x_172, x_138); x_174 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__1; x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; x_176 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__59; -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_177 = l_Lean_Name_mkStr3(x_133, x_135, x_176); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_177 = l_Lean_Name_mkStr3(x_147, x_142, x_176); x_178 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_178, 0, x_177); x_179 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_133); -x_180 = l_Lean_Name_mkStr3(x_133, x_179, x_176); +lean_inc_ref(x_147); +x_180 = l_Lean_Name_mkStr3(x_147, x_179, x_176); x_181 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_181, 0, x_180); -lean_inc_ref(x_133); -x_182 = l_Lean_Name_mkStr2(x_133, x_179); +lean_inc_ref(x_147); +x_182 = l_Lean_Name_mkStr2(x_147, x_179); x_183 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_183, 0, x_182); -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_184 = l_Lean_Name_mkStr2(x_133, x_135); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_184 = l_Lean_Name_mkStr2(x_147, x_142); x_185 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_185, 0, x_184); -lean_inc_ref(x_133); -x_186 = l_Lean_Name_mkStr1(x_133); +lean_inc_ref(x_147); +x_186 = l_Lean_Name_mkStr1(x_147); x_187 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_187, 0, x_186); -lean_inc(x_146); +lean_inc(x_135); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_187); -lean_ctor_set(x_188, 1, x_146); +lean_ctor_set(x_188, 1, x_135); x_189 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_189, 0, x_185); lean_ctor_set(x_189, 1, x_188); @@ -11901,95 +11901,95 @@ lean_ctor_set(x_192, 1, x_191); x_193 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_193, 0, x_175); lean_ctor_set(x_193, 1, x_192); -lean_inc(x_138); +lean_inc(x_137); x_194 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_194, 0, x_138); +lean_ctor_set(x_194, 0, x_137); lean_ctor_set(x_194, 1, x_171); lean_ctor_set(x_194, 2, x_173); lean_ctor_set(x_194, 3, x_193); -lean_inc(x_138); -x_195 = l_Lean_Syntax_node1(x_138, x_170, x_194); -lean_inc(x_138); -x_196 = l_Lean_Syntax_node2(x_138, x_167, x_169, x_195); +lean_inc(x_137); +x_195 = l_Lean_Syntax_node1(x_137, x_170, x_194); +lean_inc(x_137); +x_196 = l_Lean_Syntax_node2(x_137, x_167, x_169, x_195); x_197 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__37; x_198 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__38; -lean_inc(x_138); +lean_inc(x_137); x_199 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_199, 0, x_138); +lean_ctor_set(x_199, 0, x_137); lean_ctor_set(x_199, 1, x_198); -lean_inc(x_138); -x_200 = l_Lean_Syntax_node1(x_138, x_197, x_199); +lean_inc(x_137); +x_200 = l_Lean_Syntax_node1(x_137, x_197, x_199); x_201 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__7; -lean_inc(x_138); +lean_inc(x_137); x_202 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_202, 0, x_138); +lean_ctor_set(x_202, 0, x_137); lean_ctor_set(x_202, 1, x_201); -lean_inc(x_139); +lean_inc(x_141); +lean_inc(x_143); lean_inc(x_137); -lean_inc(x_138); -x_203 = l_Lean_Syntax_node1(x_138, x_137, x_139); +x_203 = l_Lean_Syntax_node1(x_137, x_143, x_141); lean_inc(x_200); +lean_inc(x_143); lean_inc(x_137); -lean_inc(x_138); -x_204 = l_Lean_Syntax_node3(x_138, x_137, x_200, x_202, x_203); +x_204 = l_Lean_Syntax_node3(x_137, x_143, x_200, x_202, x_203); x_205 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; -lean_inc(x_138); +lean_inc(x_137); x_206 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_206, 0, x_138); +lean_ctor_set(x_206, 0, x_137); lean_ctor_set(x_206, 1, x_205); -lean_inc(x_138); -x_207 = l_Lean_Syntax_node3(x_138, x_165, x_196, x_204, x_206); +lean_inc(x_137); +x_207 = l_Lean_Syntax_node3(x_137, x_165, x_196, x_204, x_206); x_208 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__14; -lean_inc(x_138); +lean_inc(x_137); x_209 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_209, 0, x_138); +lean_ctor_set(x_209, 0, x_137); lean_ctor_set(x_209, 1, x_208); x_210 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_143); -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_211 = l_Lean_Name_mkStr4(x_133, x_135, x_143, x_210); +lean_inc_ref(x_134); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_211 = l_Lean_Name_mkStr4(x_147, x_142, x_134, x_210); x_212 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_213 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; -lean_inc(x_147); +lean_inc(x_138); lean_inc(x_148); -x_214 = l_Lean_addMacroScope(x_148, x_213, x_147); +x_214 = l_Lean_addMacroScope(x_148, x_213, x_138); x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__8; x_216 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_146); +lean_inc(x_135); x_217 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_217, 0, x_216); -lean_ctor_set(x_217, 1, x_146); +lean_ctor_set(x_217, 1, x_135); x_218 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_218, 0, x_215); lean_ctor_set(x_218, 1, x_217); -lean_inc(x_138); +lean_inc(x_137); x_219 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_219, 0, x_138); +lean_ctor_set(x_219, 0, x_137); lean_ctor_set(x_219, 1, x_212); lean_ctor_set(x_219, 2, x_214); lean_ctor_set(x_219, 3, x_218); -lean_inc(x_136); +lean_inc(x_133); +lean_inc(x_143); lean_inc(x_137); -lean_inc(x_138); -x_220 = l_Lean_Syntax_node1(x_138, x_137, x_136); +x_220 = l_Lean_Syntax_node1(x_137, x_143, x_133); lean_inc(x_211); -lean_inc(x_138); -x_221 = l_Lean_Syntax_node2(x_138, x_211, x_219, x_220); +lean_inc(x_137); +x_221 = l_Lean_Syntax_node2(x_137, x_211, x_219, x_220); lean_inc_ref(x_209); lean_inc_ref(x_156); -lean_inc(x_144); +lean_inc(x_146); lean_inc_ref(x_152); -lean_inc(x_138); -x_222 = l_Lean_Syntax_node8(x_138, x_151, x_152, x_154, x_144, x_156, x_163, x_207, x_209, x_221); +lean_inc(x_137); +x_222 = l_Lean_Syntax_node8(x_137, x_151, x_152, x_154, x_146, x_156, x_163, x_207, x_209, x_221); x_223 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_224 = l_Lean_Name_mkStr4(x_133, x_135, x_176, x_223); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_224 = l_Lean_Name_mkStr4(x_147, x_142, x_176, x_223); x_225 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_135); -lean_inc_ref(x_133); -x_226 = l_Lean_Name_mkStr4(x_133, x_135, x_176, x_225); +lean_inc_ref(x_142); +lean_inc_ref(x_147); +x_226 = l_Lean_Name_mkStr4(x_147, x_142, x_176, x_225); if (lean_obj_tag(x_6) == 1) { lean_object* x_227; lean_object* x_228; @@ -11997,36 +11997,36 @@ x_227 = lean_ctor_get(x_6, 0); lean_inc(x_227); lean_dec_ref(x_6); x_228 = l_Array_mkArray1___redArg(x_227); -x_13 = x_226; -x_14 = x_176; -x_15 = x_174; -x_16 = x_133; -x_17 = x_148; -x_18 = x_136; -x_19 = x_222; +x_13 = x_133; +x_14 = x_152; +x_15 = x_134; +x_16 = x_209; +x_17 = x_135; +x_18 = x_139; +x_19 = x_137; x_20 = x_224; -x_21 = x_140; -x_22 = x_141; -x_23 = x_150; +x_21 = x_226; +x_22 = x_176; +x_23 = x_148; x_24 = x_142; -x_25 = x_143; -x_26 = x_145; -x_27 = x_146; -x_28 = x_160; -x_29 = x_156; -x_30 = x_134; -x_31 = x_135; -x_32 = x_137; -x_33 = x_138; -x_34 = x_139; -x_35 = lean_box(0); -x_36 = x_200; -x_37 = x_144; -x_38 = x_209; -x_39 = x_201; -x_40 = x_211; -x_41 = x_152; -x_42 = x_147; +x_25 = x_222; +x_26 = x_143; +x_27 = x_144; +x_28 = x_146; +x_29 = x_200; +x_30 = x_156; +x_31 = x_147; +x_32 = x_174; +x_33 = x_160; +x_34 = x_150; +x_35 = x_201; +x_36 = x_136; +x_37 = x_138; +x_38 = x_140; +x_39 = x_141; +x_40 = lean_box(0); +x_41 = x_145; +x_42 = x_211; x_43 = x_228; goto block_132; } @@ -12035,36 +12035,36 @@ else lean_object* x_229; lean_dec(x_6); x_229 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_13 = x_226; -x_14 = x_176; -x_15 = x_174; -x_16 = x_133; -x_17 = x_148; -x_18 = x_136; -x_19 = x_222; +x_13 = x_133; +x_14 = x_152; +x_15 = x_134; +x_16 = x_209; +x_17 = x_135; +x_18 = x_139; +x_19 = x_137; x_20 = x_224; -x_21 = x_140; -x_22 = x_141; -x_23 = x_150; +x_21 = x_226; +x_22 = x_176; +x_23 = x_148; x_24 = x_142; -x_25 = x_143; -x_26 = x_145; -x_27 = x_146; -x_28 = x_160; -x_29 = x_156; -x_30 = x_134; -x_31 = x_135; -x_32 = x_137; -x_33 = x_138; -x_34 = x_139; -x_35 = lean_box(0); -x_36 = x_200; -x_37 = x_144; -x_38 = x_209; -x_39 = x_201; -x_40 = x_211; -x_41 = x_152; -x_42 = x_147; +x_25 = x_222; +x_26 = x_143; +x_27 = x_144; +x_28 = x_146; +x_29 = x_200; +x_30 = x_156; +x_31 = x_147; +x_32 = x_174; +x_33 = x_160; +x_34 = x_150; +x_35 = x_201; +x_36 = x_136; +x_37 = x_138; +x_38 = x_140; +x_39 = x_141; +x_40 = lean_box(0); +x_41 = x_145; +x_42 = x_211; x_43 = x_229; goto block_132; } @@ -13361,106 +13361,106 @@ goto block_106; { 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_17 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_12); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_14); -x_18 = l_Lean_Name_mkStr4(x_14, x_11, x_12, x_17); -x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; lean_inc_ref(x_12); +x_18 = l_Lean_Name_mkStr4(x_12, x_11, x_15, x_17); +x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_14); -x_20 = l_Lean_Name_mkStr4(x_14, x_11, x_12, x_19); +lean_inc_ref(x_12); +x_20 = l_Lean_Name_mkStr4(x_12, x_11, x_15, x_19); x_21 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_22 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_15); +lean_inc(x_14); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_15); +lean_ctor_set(x_23, 0, x_14); lean_ctor_set(x_23, 1, x_21); lean_ctor_set(x_23, 2, x_22); lean_inc_ref_n(x_23, 7); -lean_inc(x_15); -x_24 = l_Lean_Syntax_node7(x_15, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); +lean_inc(x_14); +x_24 = l_Lean_Syntax_node7(x_14, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); x_25 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_12); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_14); -x_26 = l_Lean_Name_mkStr4(x_14, x_11, x_12, x_25); +lean_inc_ref(x_12); +x_26 = l_Lean_Name_mkStr4(x_12, x_11, x_15, x_25); x_27 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_15); +lean_inc(x_14); x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_15); +lean_ctor_set(x_28, 0, x_14); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_12); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_14); -x_30 = l_Lean_Name_mkStr4(x_14, x_11, x_12, x_29); +lean_inc_ref(x_12); +x_30 = l_Lean_Name_mkStr4(x_12, x_11, x_15, x_29); x_31 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; -lean_inc(x_9); +lean_inc(x_8); x_32 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_32, 0, x_9); +lean_ctor_set(x_32, 0, x_8); lean_ctor_set(x_32, 1, x_21); lean_ctor_set(x_32, 2, x_31); x_33 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_34 = lean_array_push(x_33, x_2); x_35 = lean_array_push(x_34, x_32); x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_9); +lean_ctor_set(x_36, 0, x_8); lean_ctor_set(x_36, 1, x_30); lean_ctor_set(x_36, 2, x_35); x_37 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; lean_inc_ref(x_11); -lean_inc_ref(x_14); -x_38 = l_Lean_Name_mkStr4(x_14, x_11, x_12, x_37); +lean_inc_ref(x_12); +x_38 = l_Lean_Name_mkStr4(x_12, x_11, x_15, x_37); x_39 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_40 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -x_41 = l_Lean_Name_mkStr4(x_14, x_11, x_39, x_40); +x_41 = l_Lean_Name_mkStr4(x_12, x_11, x_39, x_40); x_42 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_15); +lean_inc(x_14); x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_15); +lean_ctor_set(x_43, 0, x_14); lean_ctor_set(x_43, 1, x_42); -lean_inc(x_15); -x_44 = l_Lean_Syntax_node2(x_15, x_41, x_43, x_3); -lean_inc(x_15); -x_45 = l_Lean_Syntax_node1(x_15, x_21, x_44); +lean_inc(x_14); +x_44 = l_Lean_Syntax_node2(x_14, x_41, x_43, x_3); +lean_inc(x_14); +x_45 = l_Lean_Syntax_node1(x_14, x_21, x_44); lean_inc_ref(x_23); -lean_inc(x_15); -x_46 = l_Lean_Syntax_node2(x_15, x_38, x_23, x_45); -lean_inc(x_15); -x_47 = l_Lean_Syntax_node5(x_15, x_26, x_28, x_36, x_46, x_13, x_23); -x_48 = l_Lean_Syntax_node2(x_15, x_18, x_24, x_47); +lean_inc(x_14); +x_46 = l_Lean_Syntax_node2(x_14, x_38, x_23, x_45); +lean_inc(x_14); +x_47 = l_Lean_Syntax_node5(x_14, x_26, x_28, x_36, x_46, x_9, x_23); +x_48 = l_Lean_Syntax_node2(x_14, x_18, x_24, x_47); lean_inc(x_48); x_49 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___boxed), 4, 1); lean_closure_set(x_49, 0, x_48); -x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_10, x_8); +x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_13, x_10); return x_50; } block_82: { lean_object* x_62; -x_62 = l_Lean_Elab_Command_getRef___redArg(x_53); +x_62 = l_Lean_Elab_Command_getRef___redArg(x_57); if (lean_obj_tag(x_62) == 0) { lean_object* x_63; lean_object* x_64; x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); lean_dec_ref(x_62); -x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_53); +x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_57); 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; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_dec_ref(x_64); -x_65 = lean_ctor_get(x_53, 5); +x_65 = lean_ctor_get(x_57, 5); x_66 = l_Lean_mkOptionalNode(x_61); x_67 = l_Lake_DSL_elabConfig___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__2___closed__0; -x_68 = lean_array_push(x_67, x_55); -x_69 = lean_array_push(x_68, x_54); +x_68 = lean_array_push(x_67, x_59); +x_69 = lean_array_push(x_68, x_52); x_70 = lean_array_push(x_69, x_66); x_71 = lean_box(2); x_72 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_57); +lean_ctor_set(x_72, 1, x_58); lean_ctor_set(x_72, 2, x_70); x_73 = 0; x_74 = l_Lean_SourceInfo_fromRef(x_63, x_73); @@ -13468,29 +13468,29 @@ lean_dec(x_63); if (lean_obj_tag(x_65) == 0) { lean_object* x_75; -x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_52); +x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_56); lean_dec_ref(x_75); -x_8 = x_52; -x_9 = x_71; -x_10 = x_53; -x_11 = x_56; -x_12 = x_58; -x_13 = x_72; -x_14 = x_60; -x_15 = x_74; +x_8 = x_71; +x_9 = x_72; +x_10 = x_56; +x_11 = x_55; +x_12 = x_54; +x_13 = x_57; +x_14 = x_74; +x_15 = x_60; x_16 = lean_box(0); goto block_51; } else { -x_8 = x_52; -x_9 = x_71; -x_10 = x_53; -x_11 = x_56; -x_12 = x_58; -x_13 = x_72; -x_14 = x_60; -x_15 = x_74; +x_8 = x_71; +x_9 = x_72; +x_10 = x_56; +x_11 = x_55; +x_12 = x_54; +x_13 = x_57; +x_14 = x_74; +x_15 = x_60; x_16 = lean_box(0); goto block_51; } @@ -13501,12 +13501,12 @@ uint8_t x_76; lean_dec(x_63); lean_dec(x_61); lean_dec_ref(x_60); -lean_dec_ref(x_58); -lean_dec(x_57); -lean_dec_ref(x_56); -lean_dec(x_55); -lean_dec(x_54); -lean_dec_ref(x_53); +lean_dec(x_59); +lean_dec(x_58); +lean_dec_ref(x_57); +lean_dec(x_56); +lean_dec_ref(x_55); +lean_dec_ref(x_54); lean_dec(x_52); lean_dec(x_4); lean_dec(x_3); @@ -13533,12 +13533,12 @@ else uint8_t x_79; lean_dec(x_61); lean_dec_ref(x_60); -lean_dec_ref(x_58); -lean_dec(x_57); -lean_dec_ref(x_56); -lean_dec(x_55); -lean_dec(x_54); -lean_dec_ref(x_53); +lean_dec(x_59); +lean_dec(x_58); +lean_dec_ref(x_57); +lean_dec(x_56); +lean_dec_ref(x_55); +lean_dec_ref(x_54); lean_dec(x_52); lean_dec(x_4); lean_dec(x_3); @@ -13587,15 +13587,15 @@ if (lean_obj_tag(x_86) == 0) { lean_object* x_99; x_99 = lean_box(0); -x_52 = x_88; -x_53 = x_87; -x_54 = x_92; -x_55 = x_94; -x_56 = x_96; -x_57 = x_98; -x_58 = x_97; -x_59 = lean_box(0); -x_60 = x_95; +x_52 = x_92; +x_53 = lean_box(0); +x_54 = x_95; +x_55 = x_96; +x_56 = x_88; +x_57 = x_87; +x_58 = x_98; +x_59 = x_94; +x_60 = x_97; x_61 = x_99; goto block_82; } @@ -13605,15 +13605,15 @@ uint8_t x_100; x_100 = !lean_is_exclusive(x_86); if (x_100 == 0) { -x_52 = x_88; -x_53 = x_87; -x_54 = x_92; -x_55 = x_94; -x_56 = x_96; -x_57 = x_98; -x_58 = x_97; -x_59 = lean_box(0); -x_60 = x_95; +x_52 = x_92; +x_53 = lean_box(0); +x_54 = x_95; +x_55 = x_96; +x_56 = x_88; +x_57 = x_87; +x_58 = x_98; +x_59 = x_94; +x_60 = x_97; x_61 = x_86; goto block_82; } @@ -13625,15 +13625,15 @@ lean_inc(x_101); lean_dec(x_86); x_102 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_102, 0, x_101); -x_52 = x_88; -x_53 = x_87; -x_54 = x_92; -x_55 = x_94; -x_56 = x_96; -x_57 = x_98; -x_58 = x_97; -x_59 = lean_box(0); -x_60 = x_95; +x_52 = x_92; +x_53 = lean_box(0); +x_54 = x_95; +x_55 = x_96; +x_56 = x_88; +x_57 = x_87; +x_58 = x_98; +x_59 = x_94; +x_60 = x_97; x_61 = x_102; goto block_82; } @@ -13743,22 +13743,22 @@ lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; x_259 = lean_ctor_get(x_258, 0); lean_inc(x_259); lean_dec_ref(x_258); -lean_inc_ref(x_244); -lean_inc(x_237); -lean_inc(x_248); +lean_inc_ref(x_236); +lean_inc(x_238); +lean_inc(x_245); x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_248); -lean_ctor_set(x_260, 1, x_237); -lean_ctor_set(x_260, 2, x_244); +lean_ctor_set(x_260, 0, x_245); +lean_ctor_set(x_260, 1, x_238); +lean_ctor_set(x_260, 2, x_236); lean_inc_ref(x_260); -lean_inc(x_248); -x_261 = l_Lean_Syntax_node1(x_248, x_238, x_260); -lean_inc(x_248); -x_262 = l_Lean_Syntax_node2(x_248, x_245, x_242, x_260); -x_263 = l_Lean_Syntax_node2(x_248, x_243, x_261, x_262); +lean_inc(x_245); +x_261 = l_Lean_Syntax_node1(x_245, x_248, x_260); +lean_inc(x_245); +x_262 = l_Lean_Syntax_node2(x_245, x_239, x_237, x_260); +x_263 = l_Lean_Syntax_node2(x_245, x_250, x_261, x_262); x_264 = lean_unsigned_to_nat(2u); x_265 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_266 = lean_array_push(x_265, x_247); +x_266 = lean_array_push(x_265, x_242); x_267 = lean_array_push(x_266, x_263); x_268 = l_Lake_DSL_expandAttrs(x_6); x_269 = l_Array_append___redArg(x_267, x_268); @@ -13772,21 +13772,21 @@ lean_dec(x_10); x_272 = lean_ctor_get(x_271, 0); lean_inc(x_272); lean_dec_ref(x_271); -x_132 = x_269; -x_133 = x_236; -x_134 = x_237; -x_135 = x_253; +x_132 = x_236; +x_133 = x_238; +x_134 = x_253; +x_135 = x_240; x_136 = x_259; -x_137 = x_239; -x_138 = x_240; -x_139 = x_241; -x_140 = x_264; -x_141 = x_244; +x_137 = x_241; +x_138 = x_243; +x_139 = x_244; +x_140 = x_270; +x_141 = x_269; x_142 = x_246; -x_143 = x_270; +x_143 = x_247; x_144 = x_257; x_145 = x_249; -x_146 = x_250; +x_146 = x_264; x_147 = x_272; x_148 = lean_box(0); goto block_229; @@ -13798,21 +13798,21 @@ lean_dec(x_10); x_273 = lean_ctor_get(x_234, 0); lean_inc(x_273); lean_dec_ref(x_234); -x_132 = x_269; -x_133 = x_236; -x_134 = x_237; -x_135 = x_253; +x_132 = x_236; +x_133 = x_238; +x_134 = x_253; +x_135 = x_240; x_136 = x_259; -x_137 = x_239; -x_138 = x_240; -x_139 = x_241; -x_140 = x_264; -x_141 = x_244; +x_137 = x_241; +x_138 = x_243; +x_139 = x_244; +x_140 = x_270; +x_141 = x_269; x_142 = x_246; -x_143 = x_270; +x_143 = x_247; x_144 = x_257; x_145 = x_249; -x_146 = x_250; +x_146 = x_264; x_147 = x_273; x_148 = lean_box(0); goto block_229; @@ -13824,18 +13824,18 @@ uint8_t x_274; lean_dec(x_257); lean_dec(x_255); lean_dec(x_253); -lean_dec_ref(x_250); +lean_dec(x_250); lean_dec(x_249); lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); -lean_dec_ref(x_244); -lean_dec(x_243); +lean_dec(x_244); +lean_dec_ref(x_243); lean_dec(x_242); lean_dec(x_241); -lean_dec(x_240); -lean_dec_ref(x_239); +lean_dec_ref(x_240); +lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); lean_dec_ref(x_236); @@ -13866,18 +13866,18 @@ else uint8_t x_277; lean_dec(x_255); lean_dec(x_253); -lean_dec_ref(x_250); +lean_dec(x_250); lean_dec(x_249); lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); -lean_dec_ref(x_244); -lean_dec(x_243); +lean_dec(x_244); +lean_dec_ref(x_243); lean_dec(x_242); lean_dec(x_241); -lean_dec(x_240); -lean_dec_ref(x_239); +lean_dec_ref(x_240); +lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); lean_dec_ref(x_236); @@ -13908,18 +13908,18 @@ else { uint8_t x_280; lean_dec(x_253); -lean_dec_ref(x_250); +lean_dec(x_250); lean_dec(x_249); lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); -lean_dec_ref(x_244); -lean_dec(x_243); +lean_dec(x_244); +lean_dec_ref(x_243); lean_dec(x_242); lean_dec(x_241); -lean_dec(x_240); -lean_dec_ref(x_239); +lean_dec_ref(x_240); +lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); lean_dec_ref(x_236); @@ -13948,18 +13948,18 @@ return x_282; } else { -lean_dec_ref(x_250); +lean_dec(x_250); lean_dec(x_249); lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); -lean_dec_ref(x_244); -lean_dec(x_243); +lean_dec(x_244); +lean_dec_ref(x_243); lean_dec(x_242); lean_dec(x_241); -lean_dec(x_240); -lean_dec_ref(x_239); +lean_dec_ref(x_240); +lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); lean_dec_ref(x_236); @@ -14005,14 +14005,14 @@ x_304 = l_Lean_Syntax_node1(x_288, x_300, x_303); x_305 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_306 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_307 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_308 = l_Lean_addMacroScope(x_291, x_307, x_287); -lean_inc(x_284); +x_308 = l_Lean_addMacroScope(x_291, x_307, x_286); +lean_inc(x_289); lean_inc(x_288); x_309 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_309, 0, x_288); lean_ctor_set(x_309, 1, x_306); lean_ctor_set(x_309, 2, x_308); -lean_ctor_set(x_309, 3, x_284); +lean_ctor_set(x_309, 3, x_289); lean_inc(x_288); x_310 = l_Lean_Syntax_node2(x_288, x_305, x_309, x_303); x_311 = l_Lean_Syntax_node2(x_288, x_299, x_304, x_310); @@ -14021,41 +14021,41 @@ if (lean_obj_tag(x_234) == 0) lean_object* x_312; x_312 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_10); lean_dec_ref(x_312); -x_236 = x_297; -x_237 = x_301; -x_238 = x_300; -x_239 = x_296; -x_240 = x_286; -x_241 = x_285; -x_242 = x_290; -x_243 = x_299; -x_244 = x_302; -x_245 = x_305; -x_246 = x_284; -x_247 = x_311; -x_248 = x_294; +x_236 = x_302; +x_237 = x_284; +x_238 = x_301; +x_239 = x_305; +x_240 = x_298; +x_241 = x_290; +x_242 = x_311; +x_243 = x_296; +x_244 = x_285; +x_245 = x_294; +x_246 = x_297; +x_247 = x_287; +x_248 = x_300; x_249 = x_289; -x_250 = x_298; +x_250 = x_299; x_251 = lean_box(0); goto block_283; } else { -x_236 = x_297; -x_237 = x_301; -x_238 = x_300; -x_239 = x_296; -x_240 = x_286; -x_241 = x_285; -x_242 = x_290; -x_243 = x_299; -x_244 = x_302; -x_245 = x_305; -x_246 = x_284; -x_247 = x_311; -x_248 = x_294; +x_236 = x_302; +x_237 = x_284; +x_238 = x_301; +x_239 = x_305; +x_240 = x_298; +x_241 = x_290; +x_242 = x_311; +x_243 = x_296; +x_244 = x_285; +x_245 = x_294; +x_246 = x_297; +x_247 = x_287; +x_248 = x_300; x_249 = x_289; -x_250 = x_298; +x_250 = x_299; x_251 = lean_box(0); goto block_283; } @@ -14195,13 +14195,13 @@ x_342 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkC x_343 = lean_ctor_get(x_342, 0); lean_inc(x_343); lean_dec_ref(x_342); -x_284 = x_328; -x_285 = x_324; -x_286 = x_331; -x_287 = x_341; +x_284 = x_337; +x_285 = x_329; +x_286 = x_341; +x_287 = x_331; x_288 = x_339; -x_289 = x_329; -x_290 = x_337; +x_289 = x_328; +x_290 = x_324; x_291 = x_343; x_292 = lean_box(0); goto block_319; @@ -14214,13 +14214,13 @@ lean_inc(x_344); lean_dec_ref(x_340); x_345 = lean_ctor_get(x_234, 0); lean_inc(x_345); -x_284 = x_328; -x_285 = x_324; -x_286 = x_331; -x_287 = x_344; +x_284 = x_337; +x_285 = x_329; +x_286 = x_344; +x_287 = x_331; x_288 = x_339; -x_289 = x_329; -x_290 = x_337; +x_289 = x_328; +x_290 = x_324; x_291 = x_345; x_292 = lean_box(0); goto block_319; @@ -14417,43 +14417,43 @@ return x_364; block_131: { 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_inc_ref(x_36); -x_43 = l_Array_append___redArg(x_36, x_42); +lean_inc_ref(x_12); +x_43 = l_Array_append___redArg(x_12, x_42); lean_dec_ref(x_42); -lean_inc(x_14); -lean_inc(x_24); +lean_inc(x_16); +lean_inc(x_27); x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_24); -lean_ctor_set(x_44, 1, x_14); +lean_ctor_set(x_44, 0, x_27); +lean_ctor_set(x_44, 1, x_16); lean_ctor_set(x_44, 2, x_43); -lean_inc_n(x_12, 6); -lean_inc(x_41); -lean_inc(x_24); -x_45 = l_Lean_Syntax_node7(x_24, x_41, x_44, x_12, x_12, x_12, x_12, x_12, x_12); +lean_inc_n(x_26, 6); +lean_inc(x_36); +lean_inc(x_27); +x_45 = l_Lean_Syntax_node7(x_27, x_36, x_44, x_26, x_26, x_26, x_26, x_26, x_26); x_46 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_13); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_47 = l_Lean_Name_mkStr4(x_30, x_27, x_13, x_46); -lean_inc(x_24); +lean_inc_ref(x_14); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_47 = l_Lean_Name_mkStr4(x_20, x_25, x_14, x_46); +lean_inc(x_27); x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_24); +lean_ctor_set(x_48, 0, x_27); lean_ctor_set(x_48, 1, x_46); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_13); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_50 = l_Lean_Name_mkStr4(x_30, x_27, x_13, x_49); +lean_inc_ref(x_14); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_50 = l_Lean_Name_mkStr4(x_20, x_25, x_14, x_49); x_51 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_52 = lean_box(2); -lean_inc(x_14); +lean_inc(x_16); x_53 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_14); +lean_ctor_set(x_53, 1, x_16); lean_ctor_set(x_53, 2, x_51); -x_54 = lean_mk_empty_array_with_capacity(x_35); -lean_inc(x_33); -x_55 = lean_array_push(x_54, x_33); +x_54 = lean_mk_empty_array_with_capacity(x_41); +lean_inc(x_19); +x_55 = lean_array_push(x_54, x_19); x_56 = lean_array_push(x_55, x_53); lean_inc(x_50); x_57 = lean_alloc_ctor(1, 3, 0); @@ -14461,194 +14461,194 @@ lean_ctor_set(x_57, 0, x_52); lean_ctor_set(x_57, 1, x_50); lean_ctor_set(x_57, 2, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_13); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_59 = l_Lean_Name_mkStr4(x_30, x_27, x_13, x_58); +lean_inc_ref(x_14); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_59 = l_Lean_Name_mkStr4(x_20, x_25, x_14, x_58); x_60 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_40); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_61 = l_Lean_Name_mkStr4(x_30, x_27, x_40, x_60); -lean_inc(x_16); +lean_inc_ref(x_31); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_61 = l_Lean_Name_mkStr4(x_20, x_25, x_31, x_60); +lean_inc(x_29); lean_inc(x_61); -lean_inc(x_24); -x_62 = l_Lean_Syntax_node2(x_24, x_61, x_16, x_15); -lean_inc(x_14); -lean_inc(x_24); -x_63 = l_Lean_Syntax_node1(x_24, x_14, x_62); -lean_inc(x_12); +lean_inc(x_27); +x_62 = l_Lean_Syntax_node2(x_27, x_61, x_29, x_15); +lean_inc(x_16); +lean_inc(x_27); +x_63 = l_Lean_Syntax_node1(x_27, x_16, x_62); +lean_inc(x_26); lean_inc(x_59); -lean_inc(x_24); -x_64 = l_Lean_Syntax_node2(x_24, x_59, x_12, x_63); +lean_inc(x_27); +x_64 = l_Lean_Syntax_node2(x_27, x_59, x_26, x_63); x_65 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__60; -lean_inc_ref(x_13); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_66 = l_Lean_Name_mkStr4(x_30, x_27, x_13, x_65); +lean_inc_ref(x_14); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_66 = l_Lean_Name_mkStr4(x_20, x_25, x_14, x_65); x_67 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__1; x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__2; -lean_inc_ref(x_29); -x_69 = l_Lean_Name_mkStr3(x_29, x_20, x_68); -lean_inc(x_31); +lean_inc_ref(x_13); +x_69 = l_Lean_Name_mkStr3(x_13, x_24, x_68); +lean_inc(x_17); lean_inc(x_69); -lean_inc(x_38); -x_70 = l_Lean_addMacroScope(x_38, x_69, x_31); -lean_inc(x_18); +lean_inc(x_28); +x_70 = l_Lean_addMacroScope(x_28, x_69, x_17); +lean_inc(x_32); x_71 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_18); -lean_inc(x_22); +lean_ctor_set(x_71, 1, x_32); +lean_inc(x_37); x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_22); -lean_inc(x_24); +lean_ctor_set(x_72, 1, x_37); +lean_inc(x_27); x_73 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_73, 0, x_24); +lean_ctor_set(x_73, 0, x_27); lean_ctor_set(x_73, 1, x_67); lean_ctor_set(x_73, 2, x_70); lean_ctor_set(x_73, 3, x_72); -lean_inc(x_14); -lean_inc(x_24); -x_74 = l_Lean_Syntax_node4(x_24, x_14, x_19, x_34, x_23, x_25); -lean_inc(x_24); -x_75 = l_Lean_Syntax_node2(x_24, x_21, x_73, x_74); +lean_inc(x_16); +lean_inc(x_27); +x_74 = l_Lean_Syntax_node4(x_27, x_16, x_38, x_34, x_33, x_21); +lean_inc(x_27); +x_75 = l_Lean_Syntax_node2(x_27, x_30, x_73, x_74); x_76 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__62; x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__63; -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_78 = l_Lean_Name_mkStr4(x_30, x_27, x_76, x_77); -lean_inc_n(x_12, 2); -lean_inc(x_24); -x_79 = l_Lean_Syntax_node2(x_24, x_78, x_12, x_12); -lean_inc(x_12); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_78 = l_Lean_Name_mkStr4(x_20, x_25, x_76, x_77); +lean_inc_n(x_26, 2); +lean_inc(x_27); +x_79 = l_Lean_Syntax_node2(x_27, x_78, x_26, x_26); +lean_inc(x_26); lean_inc(x_79); -lean_inc(x_28); -lean_inc(x_66); -lean_inc(x_24); -x_80 = l_Lean_Syntax_node4(x_24, x_66, x_28, x_75, x_79, x_12); -lean_inc(x_24); -x_81 = l_Lean_Syntax_node4(x_24, x_47, x_48, x_57, x_64, x_80); lean_inc(x_39); -lean_inc(x_24); -x_82 = l_Lean_Syntax_node2(x_24, x_39, x_45, x_81); +lean_inc(x_66); +lean_inc(x_27); +x_80 = l_Lean_Syntax_node4(x_27, x_66, x_39, x_75, x_79, x_26); +lean_inc(x_27); +x_81 = l_Lean_Syntax_node4(x_27, x_47, x_48, x_57, x_64, x_80); +lean_inc(x_18); +lean_inc(x_27); +x_82 = l_Lean_Syntax_node2(x_27, x_18, x_45, x_81); x_83 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_40); -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_84 = l_Lean_Name_mkStr4(x_30, x_27, x_40, x_83); +lean_inc_ref(x_31); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_84 = l_Lean_Name_mkStr4(x_20, x_25, x_31, x_83); x_85 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_24); +lean_inc(x_27); x_86 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_86, 0, x_24); +lean_ctor_set(x_86, 0, x_27); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Syntax_SepArray_ofElems(x_37, x_26); -lean_dec_ref(x_26); -x_88 = l_Array_append___redArg(x_36, x_87); +x_87 = l_Lean_Syntax_SepArray_ofElems(x_40, x_23); +lean_dec_ref(x_23); +x_88 = l_Array_append___redArg(x_12, x_87); lean_dec_ref(x_87); -lean_inc(x_14); -lean_inc(x_24); +lean_inc(x_16); +lean_inc(x_27); x_89 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_89, 0, x_24); -lean_ctor_set(x_89, 1, x_14); +lean_ctor_set(x_89, 0, x_27); +lean_ctor_set(x_89, 1, x_16); lean_ctor_set(x_89, 2, x_88); x_90 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_24); +lean_inc(x_27); x_91 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_91, 0, x_24); +lean_ctor_set(x_91, 0, x_27); lean_ctor_set(x_91, 1, x_90); -lean_inc(x_24); -x_92 = l_Lean_Syntax_node3(x_24, x_84, x_86, x_89, x_91); -lean_inc(x_14); -lean_inc(x_24); -x_93 = l_Lean_Syntax_node1(x_24, x_14, x_92); -lean_inc_n(x_12, 6); -lean_inc(x_24); -x_94 = l_Lean_Syntax_node7(x_24, x_41, x_12, x_93, x_12, x_12, x_12, x_12, x_12); +lean_inc(x_27); +x_92 = l_Lean_Syntax_node3(x_27, x_84, x_86, x_89, x_91); +lean_inc(x_16); +lean_inc(x_27); +x_93 = l_Lean_Syntax_node1(x_27, x_16, x_92); +lean_inc_n(x_26, 6); +lean_inc(x_27); +x_94 = l_Lean_Syntax_node7(x_27, x_36, x_26, x_93, x_26, x_26, x_26, x_26, x_26); x_95 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_27); -lean_inc_ref(x_30); -x_96 = l_Lean_Name_mkStr4(x_30, x_27, x_13, x_95); +lean_inc_ref(x_25); +lean_inc_ref(x_20); +x_96 = l_Lean_Name_mkStr4(x_20, x_25, x_14, x_95); x_97 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_24); +lean_inc(x_27); x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_24); +lean_ctor_set(x_98, 0, x_27); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_100 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_31); -lean_inc(x_38); -x_101 = l_Lean_addMacroScope(x_38, x_100, x_31); -lean_inc(x_22); -lean_inc(x_24); +lean_inc(x_17); +lean_inc(x_28); +x_101 = l_Lean_addMacroScope(x_28, x_100, x_17); +lean_inc(x_37); +lean_inc(x_27); x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_24); +lean_ctor_set(x_102, 0, x_27); lean_ctor_set(x_102, 1, x_99); lean_ctor_set(x_102, 2, x_101); -lean_ctor_set(x_102, 3, x_22); -lean_inc(x_12); -lean_inc(x_24); -x_103 = l_Lean_Syntax_node2(x_24, x_50, x_102, x_12); +lean_ctor_set(x_102, 3, x_37); +lean_inc(x_26); +lean_inc(x_27); +x_103 = l_Lean_Syntax_node2(x_27, x_50, x_102, x_26); x_104 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__5; x_105 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_106 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_31); -lean_inc(x_38); -x_107 = l_Lean_addMacroScope(x_38, x_106, x_31); -x_108 = l_Lean_Name_mkStr2(x_29, x_104); +lean_inc(x_17); +lean_inc(x_28); +x_107 = l_Lean_addMacroScope(x_28, x_106, x_17); +x_108 = l_Lean_Name_mkStr2(x_13, x_104); lean_inc(x_108); x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_18); +lean_ctor_set(x_109, 1, x_32); x_110 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_110, 0, x_108); -lean_inc(x_22); +lean_inc(x_37); x_111 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_22); +lean_ctor_set(x_111, 1, x_37); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_109); lean_ctor_set(x_112, 1, x_111); -lean_inc(x_24); +lean_inc(x_27); x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_24); +lean_ctor_set(x_113, 0, x_27); lean_ctor_set(x_113, 1, x_105); lean_ctor_set(x_113, 2, x_107); lean_ctor_set(x_113, 3, x_112); -lean_inc(x_24); -x_114 = l_Lean_Syntax_node2(x_24, x_61, x_16, x_113); -lean_inc(x_14); -lean_inc(x_24); -x_115 = l_Lean_Syntax_node1(x_24, x_14, x_114); -lean_inc(x_12); -lean_inc(x_24); -x_116 = l_Lean_Syntax_node2(x_24, x_59, x_12, x_115); +lean_inc(x_27); +x_114 = l_Lean_Syntax_node2(x_27, x_61, x_29, x_113); +lean_inc(x_16); +lean_inc(x_27); +x_115 = l_Lean_Syntax_node1(x_27, x_16, x_114); +lean_inc(x_26); +lean_inc(x_27); +x_116 = l_Lean_Syntax_node2(x_27, x_59, x_26, x_115); x_117 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_118 = l_Lean_Name_mkStr4(x_30, x_27, x_40, x_117); +x_118 = l_Lean_Name_mkStr4(x_20, x_25, x_31, x_117); x_119 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_24); +lean_inc(x_27); x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_24); +lean_ctor_set(x_120, 0, x_27); lean_ctor_set(x_120, 1, x_119); x_121 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_122 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_123 = l_Lean_addMacroScope(x_38, x_122, x_31); -lean_inc(x_24); +x_123 = l_Lean_addMacroScope(x_28, x_122, x_17); +lean_inc(x_27); x_124 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_124, 0, x_24); +lean_ctor_set(x_124, 0, x_27); lean_ctor_set(x_124, 1, x_121); lean_ctor_set(x_124, 2, x_123); -lean_ctor_set(x_124, 3, x_22); -lean_inc(x_24); -x_125 = l_Lean_Syntax_node3(x_24, x_118, x_33, x_120, x_124); -lean_inc(x_12); -lean_inc(x_24); -x_126 = l_Lean_Syntax_node4(x_24, x_66, x_28, x_125, x_79, x_12); -lean_inc(x_24); -x_127 = l_Lean_Syntax_node5(x_24, x_96, x_98, x_103, x_116, x_126, x_12); -lean_inc(x_24); -x_128 = l_Lean_Syntax_node2(x_24, x_39, x_94, x_127); -x_129 = l_Lean_Syntax_node3(x_24, x_14, x_17, x_82, x_128); +lean_ctor_set(x_124, 3, x_37); +lean_inc(x_27); +x_125 = l_Lean_Syntax_node3(x_27, x_118, x_19, x_120, x_124); +lean_inc(x_26); +lean_inc(x_27); +x_126 = l_Lean_Syntax_node4(x_27, x_66, x_39, x_125, x_79, x_26); +lean_inc(x_27); +x_127 = l_Lean_Syntax_node5(x_27, x_96, x_98, x_103, x_116, x_126, x_26); +lean_inc(x_27); +x_128 = l_Lean_Syntax_node2(x_27, x_18, x_94, x_127); +x_129 = l_Lean_Syntax_node3(x_27, x_16, x_35, x_82, x_128); x_130 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_130, 0, x_129); return x_130; @@ -14658,13 +14658,13 @@ return x_130; 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; x_149 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__0; x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; -lean_inc_ref(x_141); -lean_inc(x_134); +lean_inc_ref(x_132); +lean_inc(x_133); lean_inc(x_144); x_151 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_151, 0, x_144); -lean_ctor_set(x_151, 1, x_134); -lean_ctor_set(x_151, 2, x_141); +lean_ctor_set(x_151, 1, x_133); +lean_ctor_set(x_151, 2, x_132); x_152 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; lean_inc(x_144); x_153 = lean_alloc_ctor(2, 2, 0); @@ -14682,10 +14682,10 @@ lean_inc(x_147); x_158 = l_Lean_addMacroScope(x_147, x_157, x_136); x_159 = lean_box(0); x_160 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__3; -lean_inc(x_142); +lean_inc(x_145); x_161 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_142); +lean_ctor_set(x_161, 1, x_145); lean_inc(x_144); x_162 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_162, 0, x_144); @@ -14693,15 +14693,15 @@ lean_ctor_set(x_162, 1, x_156); lean_ctor_set(x_162, 2, x_158); lean_ctor_set(x_162, 3, x_161); x_163 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_146); -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_164 = l_Lean_Name_mkStr4(x_137, x_133, x_146, x_163); +lean_inc_ref(x_135); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_164 = l_Lean_Name_mkStr4(x_138, x_142, x_135, x_163); x_165 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_146); -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_166 = l_Lean_Name_mkStr4(x_137, x_133, x_146, x_165); +lean_inc_ref(x_135); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_166 = l_Lean_Name_mkStr4(x_138, x_142, x_135, x_165); x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; lean_inc(x_144); x_168 = lean_alloc_ctor(2, 2, 0); @@ -14716,33 +14716,33 @@ x_172 = l_Lean_addMacroScope(x_147, x_171, x_136); x_173 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__1; x_174 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__59; -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_176 = l_Lean_Name_mkStr3(x_137, x_133, x_175); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_176 = l_Lean_Name_mkStr3(x_138, x_142, x_175); x_177 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_177, 0, x_176); x_178 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_137); -x_179 = l_Lean_Name_mkStr3(x_137, x_178, x_175); +lean_inc_ref(x_138); +x_179 = l_Lean_Name_mkStr3(x_138, x_178, x_175); x_180 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_180, 0, x_179); -lean_inc_ref(x_137); -x_181 = l_Lean_Name_mkStr2(x_137, x_178); +lean_inc_ref(x_138); +x_181 = l_Lean_Name_mkStr2(x_138, x_178); x_182 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_182, 0, x_181); -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_183 = l_Lean_Name_mkStr2(x_137, x_133); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_183 = l_Lean_Name_mkStr2(x_138, x_142); x_184 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_184, 0, x_183); -lean_inc_ref(x_137); -x_185 = l_Lean_Name_mkStr1(x_137); +lean_inc_ref(x_138); +x_185 = l_Lean_Name_mkStr1(x_138); x_186 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_186, 0, x_185); -lean_inc(x_142); +lean_inc(x_145); x_187 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_187, 0, x_186); -lean_ctor_set(x_187, 1, x_142); +lean_ctor_set(x_187, 1, x_145); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_184); lean_ctor_set(x_188, 1, x_187); @@ -14781,14 +14781,14 @@ lean_inc(x_144); x_201 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_201, 0, x_144); lean_ctor_set(x_201, 1, x_200); -lean_inc(x_138); -lean_inc(x_134); +lean_inc(x_143); +lean_inc(x_133); lean_inc(x_144); -x_202 = l_Lean_Syntax_node1(x_144, x_134, x_138); +x_202 = l_Lean_Syntax_node1(x_144, x_133, x_143); lean_inc(x_199); -lean_inc(x_134); +lean_inc(x_133); lean_inc(x_144); -x_203 = l_Lean_Syntax_node3(x_144, x_134, x_199, x_201, x_202); +x_203 = l_Lean_Syntax_node3(x_144, x_133, x_199, x_201, x_202); x_204 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; lean_inc(x_144); x_205 = lean_alloc_ctor(2, 2, 0); @@ -14802,10 +14802,10 @@ x_208 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_208, 0, x_144); lean_ctor_set(x_208, 1, x_207); x_209 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_146); -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_210 = l_Lean_Name_mkStr4(x_137, x_133, x_146, x_209); +lean_inc_ref(x_135); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_210 = l_Lean_Name_mkStr4(x_138, x_142, x_135, x_209); x_211 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_212 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; lean_inc(x_136); @@ -14813,10 +14813,10 @@ lean_inc(x_147); x_213 = l_Lean_addMacroScope(x_147, x_212, x_136); x_214 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__8; x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_142); +lean_inc(x_145); x_216 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_142); +lean_ctor_set(x_216, 1, x_145); x_217 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_217, 0, x_214); lean_ctor_set(x_217, 1, x_216); @@ -14826,27 +14826,27 @@ lean_ctor_set(x_218, 0, x_144); lean_ctor_set(x_218, 1, x_211); lean_ctor_set(x_218, 2, x_213); lean_ctor_set(x_218, 3, x_217); -lean_inc(x_143); -lean_inc(x_134); +lean_inc(x_140); +lean_inc(x_133); lean_inc(x_144); -x_219 = l_Lean_Syntax_node1(x_144, x_134, x_143); +x_219 = l_Lean_Syntax_node1(x_144, x_133, x_140); lean_inc(x_210); lean_inc(x_144); x_220 = l_Lean_Syntax_node2(x_144, x_210, x_218, x_219); lean_inc_ref(x_208); lean_inc_ref(x_155); -lean_inc(x_139); +lean_inc(x_137); lean_inc_ref(x_151); lean_inc(x_144); -x_221 = l_Lean_Syntax_node8(x_144, x_150, x_151, x_153, x_139, x_155, x_162, x_206, x_208, x_220); +x_221 = l_Lean_Syntax_node8(x_144, x_150, x_151, x_153, x_137, x_155, x_162, x_206, x_208, x_220); x_222 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_223 = l_Lean_Name_mkStr4(x_137, x_133, x_175, x_222); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_223 = l_Lean_Name_mkStr4(x_138, x_142, x_175, x_222); x_224 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_133); -lean_inc_ref(x_137); -x_225 = l_Lean_Name_mkStr4(x_137, x_133, x_175, x_224); +lean_inc_ref(x_142); +lean_inc_ref(x_138); +x_225 = l_Lean_Name_mkStr4(x_138, x_142, x_175, x_224); if (lean_obj_tag(x_5) == 1) { lean_object* x_226; lean_object* x_227; @@ -14854,36 +14854,36 @@ x_226 = lean_ctor_get(x_5, 0); lean_inc(x_226); lean_dec_ref(x_5); x_227 = l_Array_mkArray1___redArg(x_226); -x_12 = x_151; -x_13 = x_175; -x_14 = x_134; -x_15 = x_135; -x_16 = x_155; -x_17 = x_221; -x_18 = x_159; -x_19 = x_199; -x_20 = x_173; -x_21 = x_210; -x_22 = x_142; -x_23 = x_143; -x_24 = x_144; -x_25 = x_145; -x_26 = x_132; -x_27 = x_133; -x_28 = x_208; -x_29 = x_149; -x_30 = x_137; -x_31 = x_136; -x_32 = lean_box(0); -x_33 = x_139; -x_34 = x_138; -x_35 = x_140; -x_36 = x_141; -x_37 = x_200; -x_38 = x_147; -x_39 = x_223; -x_40 = x_146; -x_41 = x_225; +x_12 = x_132; +x_13 = x_149; +x_14 = x_175; +x_15 = x_134; +x_16 = x_133; +x_17 = x_136; +x_18 = x_223; +x_19 = x_137; +x_20 = x_138; +x_21 = x_139; +x_22 = lean_box(0); +x_23 = x_141; +x_24 = x_173; +x_25 = x_142; +x_26 = x_151; +x_27 = x_144; +x_28 = x_147; +x_29 = x_155; +x_30 = x_210; +x_31 = x_135; +x_32 = x_159; +x_33 = x_140; +x_34 = x_143; +x_35 = x_221; +x_36 = x_225; +x_37 = x_145; +x_38 = x_199; +x_39 = x_208; +x_40 = x_200; +x_41 = x_146; x_42 = x_227; goto block_131; } @@ -14892,36 +14892,36 @@ else lean_object* x_228; lean_dec(x_5); x_228 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_12 = x_151; -x_13 = x_175; -x_14 = x_134; -x_15 = x_135; -x_16 = x_155; -x_17 = x_221; -x_18 = x_159; -x_19 = x_199; -x_20 = x_173; -x_21 = x_210; -x_22 = x_142; -x_23 = x_143; -x_24 = x_144; -x_25 = x_145; -x_26 = x_132; -x_27 = x_133; -x_28 = x_208; -x_29 = x_149; -x_30 = x_137; -x_31 = x_136; -x_32 = lean_box(0); -x_33 = x_139; -x_34 = x_138; -x_35 = x_140; -x_36 = x_141; -x_37 = x_200; -x_38 = x_147; -x_39 = x_223; -x_40 = x_146; -x_41 = x_225; +x_12 = x_132; +x_13 = x_149; +x_14 = x_175; +x_15 = x_134; +x_16 = x_133; +x_17 = x_136; +x_18 = x_223; +x_19 = x_137; +x_20 = x_138; +x_21 = x_139; +x_22 = lean_box(0); +x_23 = x_141; +x_24 = x_173; +x_25 = x_142; +x_26 = x_151; +x_27 = x_144; +x_28 = x_147; +x_29 = x_155; +x_30 = x_210; +x_31 = x_135; +x_32 = x_159; +x_33 = x_140; +x_34 = x_143; +x_35 = x_221; +x_36 = x_225; +x_37 = x_145; +x_38 = x_199; +x_39 = x_208; +x_40 = x_200; +x_41 = x_146; x_42 = x_228; goto block_131; } @@ -15843,106 +15843,106 @@ goto block_106; { 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_17 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_9); -lean_inc_ref(x_14); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -x_18 = l_Lean_Name_mkStr4(x_11, x_14, x_9, x_17); +x_18 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_17); x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_9); -lean_inc_ref(x_14); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -x_20 = l_Lean_Name_mkStr4(x_11, x_14, x_9, x_19); +x_20 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_19); x_21 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_22 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_13); +lean_inc(x_8); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_13); +lean_ctor_set(x_23, 0, x_8); lean_ctor_set(x_23, 1, x_21); lean_ctor_set(x_23, 2, x_22); lean_inc_ref_n(x_23, 7); -lean_inc(x_13); -x_24 = l_Lean_Syntax_node7(x_13, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); +lean_inc(x_8); +x_24 = l_Lean_Syntax_node7(x_8, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); x_25 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_9); -lean_inc_ref(x_14); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -x_26 = l_Lean_Name_mkStr4(x_11, x_14, x_9, x_25); +x_26 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_25); x_27 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_13); +lean_inc(x_8); x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_13); +lean_ctor_set(x_28, 0, x_8); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_9); -lean_inc_ref(x_14); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -x_30 = l_Lean_Name_mkStr4(x_11, x_14, x_9, x_29); +x_30 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_29); x_31 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; -lean_inc(x_10); +lean_inc(x_14); x_32 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_32, 0, x_10); +lean_ctor_set(x_32, 0, x_14); lean_ctor_set(x_32, 1, x_21); lean_ctor_set(x_32, 2, x_31); x_33 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_34 = lean_array_push(x_33, x_2); x_35 = lean_array_push(x_34, x_32); x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_10); +lean_ctor_set(x_36, 0, x_14); lean_ctor_set(x_36, 1, x_30); lean_ctor_set(x_36, 2, x_35); x_37 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_14); +lean_inc_ref(x_15); lean_inc_ref(x_11); -x_38 = l_Lean_Name_mkStr4(x_11, x_14, x_9, x_37); +x_38 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_37); x_39 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_40 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -x_41 = l_Lean_Name_mkStr4(x_11, x_14, x_39, x_40); +x_41 = l_Lean_Name_mkStr4(x_11, x_15, x_39, x_40); x_42 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_13); +lean_inc(x_8); x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_13); +lean_ctor_set(x_43, 0, x_8); lean_ctor_set(x_43, 1, x_42); -lean_inc(x_13); -x_44 = l_Lean_Syntax_node2(x_13, x_41, x_43, x_3); -lean_inc(x_13); -x_45 = l_Lean_Syntax_node1(x_13, x_21, x_44); +lean_inc(x_8); +x_44 = l_Lean_Syntax_node2(x_8, x_41, x_43, x_3); +lean_inc(x_8); +x_45 = l_Lean_Syntax_node1(x_8, x_21, x_44); lean_inc_ref(x_23); -lean_inc(x_13); -x_46 = l_Lean_Syntax_node2(x_13, x_38, x_23, x_45); -lean_inc(x_13); -x_47 = l_Lean_Syntax_node5(x_13, x_26, x_28, x_36, x_46, x_8, x_23); -x_48 = l_Lean_Syntax_node2(x_13, x_18, x_24, x_47); +lean_inc(x_8); +x_46 = l_Lean_Syntax_node2(x_8, x_38, x_23, x_45); +lean_inc(x_8); +x_47 = l_Lean_Syntax_node5(x_8, x_26, x_28, x_36, x_46, x_9, x_23); +x_48 = l_Lean_Syntax_node2(x_8, x_18, x_24, x_47); lean_inc(x_48); x_49 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___boxed), 4, 1); lean_closure_set(x_49, 0, x_48); -x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_12, x_15); +x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_13, x_12); return x_50; } block_82: { lean_object* x_62; -x_62 = l_Lean_Elab_Command_getRef___redArg(x_55); +x_62 = l_Lean_Elab_Command_getRef___redArg(x_58); if (lean_obj_tag(x_62) == 0) { lean_object* x_63; lean_object* x_64; x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); lean_dec_ref(x_62); -x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_55); +x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_58); 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; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_dec_ref(x_64); -x_65 = lean_ctor_get(x_55, 5); +x_65 = lean_ctor_get(x_58, 5); x_66 = l_Lean_mkOptionalNode(x_61); x_67 = l_Lake_DSL_elabConfig___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__2___closed__0; -x_68 = lean_array_push(x_67, x_60); -x_69 = lean_array_push(x_68, x_57); +x_68 = lean_array_push(x_67, x_57); +x_69 = lean_array_push(x_68, x_56); x_70 = lean_array_push(x_69, x_66); x_71 = lean_box(2); x_72 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_54); +lean_ctor_set(x_72, 1, x_52); lean_ctor_set(x_72, 2, x_70); x_73 = 0; x_74 = l_Lean_SourceInfo_fromRef(x_63, x_73); @@ -15950,28 +15950,28 @@ lean_dec(x_63); if (lean_obj_tag(x_65) == 0) { lean_object* x_75; -x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_59); +x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_55); lean_dec_ref(x_75); -x_8 = x_72; -x_9 = x_52; -x_10 = x_71; -x_11 = x_53; +x_8 = x_74; +x_9 = x_72; +x_10 = x_53; +x_11 = x_54; x_12 = x_55; -x_13 = x_74; -x_14 = x_56; +x_13 = x_58; +x_14 = x_71; x_15 = x_59; x_16 = lean_box(0); goto block_51; } else { -x_8 = x_72; -x_9 = x_52; -x_10 = x_71; -x_11 = x_53; +x_8 = x_74; +x_9 = x_72; +x_10 = x_53; +x_11 = x_54; x_12 = x_55; -x_13 = x_74; -x_14 = x_56; +x_13 = x_58; +x_14 = x_71; x_15 = x_59; x_16 = lean_box(0); goto block_51; @@ -15982,14 +15982,14 @@ else uint8_t x_76; lean_dec(x_63); lean_dec(x_61); -lean_dec(x_60); -lean_dec(x_59); +lean_dec_ref(x_59); +lean_dec_ref(x_58); lean_dec(x_57); -lean_dec_ref(x_56); -lean_dec_ref(x_55); -lean_dec(x_54); +lean_dec(x_56); +lean_dec(x_55); +lean_dec_ref(x_54); lean_dec_ref(x_53); -lean_dec_ref(x_52); +lean_dec(x_52); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -16014,14 +16014,14 @@ else { uint8_t x_79; lean_dec(x_61); -lean_dec(x_60); -lean_dec(x_59); +lean_dec_ref(x_59); +lean_dec_ref(x_58); lean_dec(x_57); -lean_dec_ref(x_56); -lean_dec_ref(x_55); -lean_dec(x_54); +lean_dec(x_56); +lean_dec(x_55); +lean_dec_ref(x_54); lean_dec_ref(x_53); -lean_dec_ref(x_52); +lean_dec(x_52); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -16069,15 +16069,15 @@ if (lean_obj_tag(x_86) == 0) { lean_object* x_99; x_99 = lean_box(0); -x_52 = x_97; -x_53 = x_95; -x_54 = x_98; -x_55 = x_87; -x_56 = x_96; -x_57 = x_92; -x_58 = lean_box(0); -x_59 = x_88; -x_60 = x_94; +x_52 = x_98; +x_53 = x_97; +x_54 = x_95; +x_55 = x_88; +x_56 = x_92; +x_57 = x_94; +x_58 = x_87; +x_59 = x_96; +x_60 = lean_box(0); x_61 = x_99; goto block_82; } @@ -16087,15 +16087,15 @@ uint8_t x_100; x_100 = !lean_is_exclusive(x_86); if (x_100 == 0) { -x_52 = x_97; -x_53 = x_95; -x_54 = x_98; -x_55 = x_87; -x_56 = x_96; -x_57 = x_92; -x_58 = lean_box(0); -x_59 = x_88; -x_60 = x_94; +x_52 = x_98; +x_53 = x_97; +x_54 = x_95; +x_55 = x_88; +x_56 = x_92; +x_57 = x_94; +x_58 = x_87; +x_59 = x_96; +x_60 = lean_box(0); x_61 = x_86; goto block_82; } @@ -16107,15 +16107,15 @@ lean_inc(x_101); lean_dec(x_86); x_102 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_102, 0, x_101); -x_52 = x_97; -x_53 = x_95; -x_54 = x_98; -x_55 = x_87; -x_56 = x_96; -x_57 = x_92; -x_58 = lean_box(0); -x_59 = x_88; -x_60 = x_94; +x_52 = x_98; +x_53 = x_97; +x_54 = x_95; +x_55 = x_88; +x_56 = x_92; +x_57 = x_94; +x_58 = x_87; +x_59 = x_96; +x_60 = lean_box(0); x_61 = x_102; goto block_82; } @@ -16225,22 +16225,22 @@ lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; x_259 = lean_ctor_get(x_258, 0); lean_inc(x_259); lean_dec_ref(x_258); -lean_inc_ref(x_249); -lean_inc(x_240); -lean_inc(x_245); +lean_inc_ref(x_241); +lean_inc(x_236); +lean_inc(x_244); x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_245); -lean_ctor_set(x_260, 1, x_240); -lean_ctor_set(x_260, 2, x_249); +lean_ctor_set(x_260, 0, x_244); +lean_ctor_set(x_260, 1, x_236); +lean_ctor_set(x_260, 2, x_241); lean_inc_ref(x_260); -lean_inc(x_245); -x_261 = l_Lean_Syntax_node1(x_245, x_236, x_260); -lean_inc(x_245); -x_262 = l_Lean_Syntax_node2(x_245, x_250, x_247, x_260); -x_263 = l_Lean_Syntax_node2(x_245, x_244, x_261, x_262); +lean_inc(x_244); +x_261 = l_Lean_Syntax_node1(x_244, x_240, x_260); +lean_inc(x_244); +x_262 = l_Lean_Syntax_node2(x_244, x_245, x_238, x_260); +x_263 = l_Lean_Syntax_node2(x_244, x_237, x_261, x_262); x_264 = lean_unsigned_to_nat(2u); x_265 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_266 = lean_array_push(x_265, x_237); +x_266 = lean_array_push(x_265, x_248); x_267 = lean_array_push(x_266, x_263); x_268 = l_Lake_DSL_expandAttrs(x_6); x_269 = l_Array_append___redArg(x_267, x_268); @@ -16254,21 +16254,21 @@ lean_dec(x_10); x_272 = lean_ctor_get(x_271, 0); lean_inc(x_272); lean_dec_ref(x_271); -x_132 = x_259; -x_133 = x_238; -x_134 = x_239; -x_135 = x_269; -x_136 = x_240; -x_137 = x_241; -x_138 = x_242; -x_139 = x_243; -x_140 = x_253; -x_141 = x_246; -x_142 = x_257; -x_143 = x_264; -x_144 = x_270; +x_132 = x_236; +x_133 = x_259; +x_134 = x_269; +x_135 = x_270; +x_136 = x_239; +x_137 = x_264; +x_138 = x_257; +x_139 = x_253; +x_140 = x_241; +x_141 = x_242; +x_142 = x_243; +x_143 = x_246; +x_144 = x_247; x_145 = x_249; -x_146 = x_248; +x_146 = x_250; x_147 = x_272; x_148 = lean_box(0); goto block_229; @@ -16280,21 +16280,21 @@ lean_dec(x_10); x_273 = lean_ctor_get(x_234, 0); lean_inc(x_273); lean_dec_ref(x_234); -x_132 = x_259; -x_133 = x_238; -x_134 = x_239; -x_135 = x_269; -x_136 = x_240; -x_137 = x_241; -x_138 = x_242; -x_139 = x_243; -x_140 = x_253; -x_141 = x_246; -x_142 = x_257; -x_143 = x_264; -x_144 = x_270; +x_132 = x_236; +x_133 = x_259; +x_134 = x_269; +x_135 = x_270; +x_136 = x_239; +x_137 = x_264; +x_138 = x_257; +x_139 = x_253; +x_140 = x_241; +x_141 = x_242; +x_142 = x_243; +x_143 = x_246; +x_144 = x_247; x_145 = x_249; -x_146 = x_248; +x_146 = x_250; x_147 = x_273; x_148 = lean_box(0); goto block_229; @@ -16307,18 +16307,18 @@ lean_dec(x_257); lean_dec(x_255); lean_dec(x_253); lean_dec(x_250); -lean_dec_ref(x_249); -lean_dec_ref(x_248); +lean_dec(x_249); +lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); lean_dec(x_244); -lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec_ref(x_243); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); -lean_dec(x_239); -lean_dec_ref(x_238); +lean_dec_ref(x_239); +lean_dec(x_238); lean_dec(x_237); lean_dec(x_236); lean_dec(x_234); @@ -16349,18 +16349,18 @@ uint8_t x_277; lean_dec(x_255); lean_dec(x_253); lean_dec(x_250); -lean_dec_ref(x_249); -lean_dec_ref(x_248); +lean_dec(x_249); +lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); lean_dec(x_244); -lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec_ref(x_243); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); -lean_dec(x_239); -lean_dec_ref(x_238); +lean_dec_ref(x_239); +lean_dec(x_238); lean_dec(x_237); lean_dec(x_236); lean_dec(x_234); @@ -16391,18 +16391,18 @@ else uint8_t x_280; lean_dec(x_253); lean_dec(x_250); -lean_dec_ref(x_249); -lean_dec_ref(x_248); +lean_dec(x_249); +lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); lean_dec(x_244); -lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec_ref(x_243); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); -lean_dec(x_239); -lean_dec_ref(x_238); +lean_dec_ref(x_239); +lean_dec(x_238); lean_dec(x_237); lean_dec(x_236); lean_dec(x_234); @@ -16431,18 +16431,18 @@ return x_282; else { lean_dec(x_250); -lean_dec_ref(x_249); -lean_dec_ref(x_248); +lean_dec(x_249); +lean_dec(x_248); lean_dec(x_247); -lean_dec(x_246); +lean_dec_ref(x_246); lean_dec(x_245); lean_dec(x_244); -lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec_ref(x_243); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); -lean_dec(x_239); -lean_dec_ref(x_238); +lean_dec_ref(x_239); +lean_dec(x_238); lean_dec(x_237); lean_dec(x_236); lean_dec(x_234); @@ -16476,68 +16476,68 @@ x_299 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_300 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_301 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_302 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_285); +lean_inc(x_290); x_303 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_303, 0, x_285); +lean_ctor_set(x_303, 0, x_290); lean_ctor_set(x_303, 1, x_301); lean_ctor_set(x_303, 2, x_302); lean_inc_ref(x_303); -lean_inc(x_285); -x_304 = l_Lean_Syntax_node1(x_285, x_300, x_303); +lean_inc(x_290); +x_304 = l_Lean_Syntax_node1(x_290, x_300, x_303); x_305 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_306 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_307 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; x_308 = l_Lean_addMacroScope(x_291, x_307, x_288); -lean_inc(x_289); -lean_inc(x_285); +lean_inc(x_284); +lean_inc(x_290); x_309 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_309, 0, x_285); +lean_ctor_set(x_309, 0, x_290); lean_ctor_set(x_309, 1, x_306); lean_ctor_set(x_309, 2, x_308); -lean_ctor_set(x_309, 3, x_289); -lean_inc(x_285); -x_310 = l_Lean_Syntax_node2(x_285, x_305, x_309, x_303); -x_311 = l_Lean_Syntax_node2(x_285, x_299, x_304, x_310); +lean_ctor_set(x_309, 3, x_284); +lean_inc(x_290); +x_310 = l_Lean_Syntax_node2(x_290, x_305, x_309, x_303); +x_311 = l_Lean_Syntax_node2(x_290, x_299, x_304, x_310); if (lean_obj_tag(x_234) == 0) { lean_object* x_312; x_312 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_10); lean_dec_ref(x_312); -x_236 = x_300; -x_237 = x_311; -x_238 = x_298; -x_239 = x_287; -x_240 = x_301; -x_241 = x_289; -x_242 = x_297; -x_243 = x_290; -x_244 = x_299; -x_245 = x_294; -x_246 = x_284; +x_236 = x_301; +x_237 = x_299; +x_238 = x_285; +x_239 = x_296; +x_240 = x_300; +x_241 = x_302; +x_242 = x_284; +x_243 = x_297; +x_244 = x_294; +x_245 = x_305; +x_246 = x_298; x_247 = x_286; -x_248 = x_296; -x_249 = x_302; -x_250 = x_305; +x_248 = x_311; +x_249 = x_287; +x_250 = x_289; x_251 = lean_box(0); goto block_283; } else { -x_236 = x_300; -x_237 = x_311; -x_238 = x_298; -x_239 = x_287; -x_240 = x_301; -x_241 = x_289; -x_242 = x_297; -x_243 = x_290; -x_244 = x_299; -x_245 = x_294; -x_246 = x_284; +x_236 = x_301; +x_237 = x_299; +x_238 = x_285; +x_239 = x_296; +x_240 = x_300; +x_241 = x_302; +x_242 = x_284; +x_243 = x_297; +x_244 = x_294; +x_245 = x_305; +x_246 = x_298; x_247 = x_286; -x_248 = x_296; -x_249 = x_302; -x_250 = x_305; +x_248 = x_311; +x_249 = x_287; +x_250 = x_289; x_251 = lean_box(0); goto block_283; } @@ -16677,13 +16677,13 @@ x_342 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkC x_343 = lean_ctor_get(x_342, 0); lean_inc(x_343); lean_dec_ref(x_342); -x_284 = x_331; -x_285 = x_339; -x_286 = x_337; -x_287 = x_324; +x_284 = x_328; +x_285 = x_337; +x_286 = x_329; +x_287 = x_331; x_288 = x_341; -x_289 = x_328; -x_290 = x_329; +x_289 = x_324; +x_290 = x_339; x_291 = x_343; x_292 = lean_box(0); goto block_319; @@ -16696,13 +16696,13 @@ lean_inc(x_344); lean_dec_ref(x_340); x_345 = lean_ctor_get(x_234, 0); lean_inc(x_345); -x_284 = x_331; -x_285 = x_339; -x_286 = x_337; -x_287 = x_324; +x_284 = x_328; +x_285 = x_337; +x_286 = x_329; +x_287 = x_331; x_288 = x_344; -x_289 = x_328; -x_290 = x_329; +x_289 = x_324; +x_290 = x_339; x_291 = x_345; x_292 = lean_box(0); goto block_319; @@ -16899,43 +16899,43 @@ return x_364; block_131: { 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_inc_ref(x_23); -x_43 = l_Array_append___redArg(x_23, x_42); +lean_inc_ref(x_37); +x_43 = l_Array_append___redArg(x_37, x_42); lean_dec_ref(x_42); -lean_inc(x_13); -lean_inc(x_34); +lean_inc(x_14); +lean_inc(x_21); x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_34); -lean_ctor_set(x_44, 1, x_13); +lean_ctor_set(x_44, 0, x_21); +lean_ctor_set(x_44, 1, x_14); lean_ctor_set(x_44, 2, x_43); -lean_inc_n(x_27, 6); -lean_inc(x_40); -lean_inc(x_34); -x_45 = l_Lean_Syntax_node7(x_34, x_40, x_44, x_27, x_27, x_27, x_27, x_27, x_27); +lean_inc_n(x_30, 6); +lean_inc(x_19); +lean_inc(x_21); +x_45 = l_Lean_Syntax_node7(x_21, x_19, x_44, x_30, x_30, x_30, x_30, x_30, x_30); x_46 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_18); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_47 = l_Lean_Name_mkStr4(x_22, x_14, x_18, x_46); -lean_inc(x_34); +lean_inc_ref(x_39); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_47 = l_Lean_Name_mkStr4(x_34, x_23, x_39, x_46); +lean_inc(x_21); x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_34); +lean_ctor_set(x_48, 0, x_21); lean_ctor_set(x_48, 1, x_46); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_18); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_50 = l_Lean_Name_mkStr4(x_22, x_14, x_18, x_49); +lean_inc_ref(x_39); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_50 = l_Lean_Name_mkStr4(x_34, x_23, x_39, x_49); x_51 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_52 = lean_box(2); -lean_inc(x_13); +lean_inc(x_14); x_53 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_13); +lean_ctor_set(x_53, 1, x_14); lean_ctor_set(x_53, 2, x_51); x_54 = lean_mk_empty_array_with_capacity(x_20); -lean_inc(x_12); -x_55 = lean_array_push(x_54, x_12); +lean_inc(x_41); +x_55 = lean_array_push(x_54, x_41); x_56 = lean_array_push(x_55, x_53); lean_inc(x_50); x_57 = lean_alloc_ctor(1, 3, 0); @@ -16943,194 +16943,194 @@ lean_ctor_set(x_57, 0, x_52); lean_ctor_set(x_57, 1, x_50); lean_ctor_set(x_57, 2, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_18); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_59 = l_Lean_Name_mkStr4(x_22, x_14, x_18, x_58); +lean_inc_ref(x_39); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_59 = l_Lean_Name_mkStr4(x_34, x_23, x_39, x_58); x_60 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_29); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_61 = l_Lean_Name_mkStr4(x_22, x_14, x_29, x_60); -lean_inc(x_37); +lean_inc_ref(x_27); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_61 = l_Lean_Name_mkStr4(x_34, x_23, x_27, x_60); +lean_inc(x_16); lean_inc(x_61); -lean_inc(x_34); -x_62 = l_Lean_Syntax_node2(x_34, x_61, x_37, x_33); -lean_inc(x_13); -lean_inc(x_34); -x_63 = l_Lean_Syntax_node1(x_34, x_13, x_62); -lean_inc(x_27); +lean_inc(x_21); +x_62 = l_Lean_Syntax_node2(x_21, x_61, x_16, x_22); +lean_inc(x_14); +lean_inc(x_21); +x_63 = l_Lean_Syntax_node1(x_21, x_14, x_62); +lean_inc(x_30); lean_inc(x_59); -lean_inc(x_34); -x_64 = l_Lean_Syntax_node2(x_34, x_59, x_27, x_63); +lean_inc(x_21); +x_64 = l_Lean_Syntax_node2(x_21, x_59, x_30, x_63); x_65 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__60; -lean_inc_ref(x_18); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_66 = l_Lean_Name_mkStr4(x_22, x_14, x_18, x_65); +lean_inc_ref(x_39); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_66 = l_Lean_Name_mkStr4(x_34, x_23, x_39, x_65); x_67 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__1; x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__2; -lean_inc_ref(x_38); -x_69 = l_Lean_Name_mkStr3(x_38, x_24, x_68); -lean_inc(x_28); +lean_inc_ref(x_36); +x_69 = l_Lean_Name_mkStr3(x_36, x_32, x_68); +lean_inc(x_15); lean_inc(x_69); -lean_inc(x_16); -x_70 = l_Lean_addMacroScope(x_16, x_69, x_28); -lean_inc(x_30); +lean_inc(x_31); +x_70 = l_Lean_addMacroScope(x_31, x_69, x_15); +lean_inc(x_12); x_71 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_30); -lean_inc(x_32); +lean_ctor_set(x_71, 1, x_12); +lean_inc(x_24); x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_32); -lean_inc(x_34); +lean_ctor_set(x_72, 1, x_24); +lean_inc(x_21); x_73 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_73, 0, x_34); +lean_ctor_set(x_73, 0, x_21); lean_ctor_set(x_73, 1, x_67); lean_ctor_set(x_73, 2, x_70); lean_ctor_set(x_73, 3, x_72); -lean_inc(x_13); -lean_inc(x_34); -x_74 = l_Lean_Syntax_node4(x_34, x_13, x_41, x_19, x_21, x_17); -lean_inc(x_34); -x_75 = l_Lean_Syntax_node2(x_34, x_39, x_73, x_74); +lean_inc(x_14); +lean_inc(x_21); +x_74 = l_Lean_Syntax_node4(x_21, x_14, x_25, x_29, x_33, x_40); +lean_inc(x_21); +x_75 = l_Lean_Syntax_node2(x_21, x_38, x_73, x_74); x_76 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__62; x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__63; -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_78 = l_Lean_Name_mkStr4(x_22, x_14, x_76, x_77); -lean_inc_n(x_27, 2); -lean_inc(x_34); -x_79 = l_Lean_Syntax_node2(x_34, x_78, x_27, x_27); -lean_inc(x_27); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_78 = l_Lean_Name_mkStr4(x_34, x_23, x_76, x_77); +lean_inc_n(x_30, 2); +lean_inc(x_21); +x_79 = l_Lean_Syntax_node2(x_21, x_78, x_30, x_30); +lean_inc(x_30); lean_inc(x_79); -lean_inc(x_35); +lean_inc(x_13); lean_inc(x_66); -lean_inc(x_34); -x_80 = l_Lean_Syntax_node4(x_34, x_66, x_35, x_75, x_79, x_27); -lean_inc(x_34); -x_81 = l_Lean_Syntax_node4(x_34, x_47, x_48, x_57, x_64, x_80); -lean_inc(x_15); -lean_inc(x_34); -x_82 = l_Lean_Syntax_node2(x_34, x_15, x_45, x_81); +lean_inc(x_21); +x_80 = l_Lean_Syntax_node4(x_21, x_66, x_13, x_75, x_79, x_30); +lean_inc(x_21); +x_81 = l_Lean_Syntax_node4(x_21, x_47, x_48, x_57, x_64, x_80); +lean_inc(x_28); +lean_inc(x_21); +x_82 = l_Lean_Syntax_node2(x_21, x_28, x_45, x_81); x_83 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_29); -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_84 = l_Lean_Name_mkStr4(x_22, x_14, x_29, x_83); +lean_inc_ref(x_27); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_84 = l_Lean_Name_mkStr4(x_34, x_23, x_27, x_83); x_85 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_34); +lean_inc(x_21); x_86 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_86, 0, x_34); +lean_ctor_set(x_86, 0, x_21); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Syntax_SepArray_ofElems(x_36, x_31); -lean_dec_ref(x_31); -x_88 = l_Array_append___redArg(x_23, x_87); +x_87 = l_Lean_Syntax_SepArray_ofElems(x_18, x_17); +lean_dec_ref(x_17); +x_88 = l_Array_append___redArg(x_37, x_87); lean_dec_ref(x_87); -lean_inc(x_13); -lean_inc(x_34); +lean_inc(x_14); +lean_inc(x_21); x_89 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_89, 0, x_34); -lean_ctor_set(x_89, 1, x_13); +lean_ctor_set(x_89, 0, x_21); +lean_ctor_set(x_89, 1, x_14); lean_ctor_set(x_89, 2, x_88); x_90 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_34); +lean_inc(x_21); x_91 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_91, 0, x_34); +lean_ctor_set(x_91, 0, x_21); lean_ctor_set(x_91, 1, x_90); -lean_inc(x_34); -x_92 = l_Lean_Syntax_node3(x_34, x_84, x_86, x_89, x_91); -lean_inc(x_13); -lean_inc(x_34); -x_93 = l_Lean_Syntax_node1(x_34, x_13, x_92); -lean_inc_n(x_27, 6); -lean_inc(x_34); -x_94 = l_Lean_Syntax_node7(x_34, x_40, x_27, x_93, x_27, x_27, x_27, x_27, x_27); +lean_inc(x_21); +x_92 = l_Lean_Syntax_node3(x_21, x_84, x_86, x_89, x_91); +lean_inc(x_14); +lean_inc(x_21); +x_93 = l_Lean_Syntax_node1(x_21, x_14, x_92); +lean_inc_n(x_30, 6); +lean_inc(x_21); +x_94 = l_Lean_Syntax_node7(x_21, x_19, x_30, x_93, x_30, x_30, x_30, x_30, x_30); x_95 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_14); -lean_inc_ref(x_22); -x_96 = l_Lean_Name_mkStr4(x_22, x_14, x_18, x_95); +lean_inc_ref(x_23); +lean_inc_ref(x_34); +x_96 = l_Lean_Name_mkStr4(x_34, x_23, x_39, x_95); x_97 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_34); +lean_inc(x_21); x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_34); +lean_ctor_set(x_98, 0, x_21); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_100 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_28); -lean_inc(x_16); -x_101 = l_Lean_addMacroScope(x_16, x_100, x_28); -lean_inc(x_32); -lean_inc(x_34); +lean_inc(x_15); +lean_inc(x_31); +x_101 = l_Lean_addMacroScope(x_31, x_100, x_15); +lean_inc(x_24); +lean_inc(x_21); x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_34); +lean_ctor_set(x_102, 0, x_21); lean_ctor_set(x_102, 1, x_99); lean_ctor_set(x_102, 2, x_101); -lean_ctor_set(x_102, 3, x_32); -lean_inc(x_27); -lean_inc(x_34); -x_103 = l_Lean_Syntax_node2(x_34, x_50, x_102, x_27); +lean_ctor_set(x_102, 3, x_24); +lean_inc(x_30); +lean_inc(x_21); +x_103 = l_Lean_Syntax_node2(x_21, x_50, x_102, x_30); x_104 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__5; x_105 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_106 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_28); -lean_inc(x_16); -x_107 = l_Lean_addMacroScope(x_16, x_106, x_28); -x_108 = l_Lean_Name_mkStr2(x_38, x_104); +lean_inc(x_15); +lean_inc(x_31); +x_107 = l_Lean_addMacroScope(x_31, x_106, x_15); +x_108 = l_Lean_Name_mkStr2(x_36, x_104); lean_inc(x_108); x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_30); +lean_ctor_set(x_109, 1, x_12); x_110 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_110, 0, x_108); -lean_inc(x_32); +lean_inc(x_24); x_111 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_32); +lean_ctor_set(x_111, 1, x_24); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_109); lean_ctor_set(x_112, 1, x_111); -lean_inc(x_34); +lean_inc(x_21); x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_34); +lean_ctor_set(x_113, 0, x_21); lean_ctor_set(x_113, 1, x_105); lean_ctor_set(x_113, 2, x_107); lean_ctor_set(x_113, 3, x_112); -lean_inc(x_34); -x_114 = l_Lean_Syntax_node2(x_34, x_61, x_37, x_113); -lean_inc(x_13); -lean_inc(x_34); -x_115 = l_Lean_Syntax_node1(x_34, x_13, x_114); -lean_inc(x_27); -lean_inc(x_34); -x_116 = l_Lean_Syntax_node2(x_34, x_59, x_27, x_115); +lean_inc(x_21); +x_114 = l_Lean_Syntax_node2(x_21, x_61, x_16, x_113); +lean_inc(x_14); +lean_inc(x_21); +x_115 = l_Lean_Syntax_node1(x_21, x_14, x_114); +lean_inc(x_30); +lean_inc(x_21); +x_116 = l_Lean_Syntax_node2(x_21, x_59, x_30, x_115); x_117 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_118 = l_Lean_Name_mkStr4(x_22, x_14, x_29, x_117); +x_118 = l_Lean_Name_mkStr4(x_34, x_23, x_27, x_117); x_119 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_34); +lean_inc(x_21); x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_34); +lean_ctor_set(x_120, 0, x_21); lean_ctor_set(x_120, 1, x_119); x_121 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_122 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_123 = l_Lean_addMacroScope(x_16, x_122, x_28); -lean_inc(x_34); +x_123 = l_Lean_addMacroScope(x_31, x_122, x_15); +lean_inc(x_21); x_124 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_124, 0, x_34); +lean_ctor_set(x_124, 0, x_21); lean_ctor_set(x_124, 1, x_121); lean_ctor_set(x_124, 2, x_123); -lean_ctor_set(x_124, 3, x_32); -lean_inc(x_34); -x_125 = l_Lean_Syntax_node3(x_34, x_118, x_12, x_120, x_124); -lean_inc(x_27); -lean_inc(x_34); -x_126 = l_Lean_Syntax_node4(x_34, x_66, x_35, x_125, x_79, x_27); -lean_inc(x_34); -x_127 = l_Lean_Syntax_node5(x_34, x_96, x_98, x_103, x_116, x_126, x_27); -lean_inc(x_34); -x_128 = l_Lean_Syntax_node2(x_34, x_15, x_94, x_127); -x_129 = l_Lean_Syntax_node3(x_34, x_13, x_25, x_82, x_128); +lean_ctor_set(x_124, 3, x_24); +lean_inc(x_21); +x_125 = l_Lean_Syntax_node3(x_21, x_118, x_41, x_120, x_124); +lean_inc(x_30); +lean_inc(x_21); +x_126 = l_Lean_Syntax_node4(x_21, x_66, x_13, x_125, x_79, x_30); +lean_inc(x_21); +x_127 = l_Lean_Syntax_node5(x_21, x_96, x_98, x_103, x_116, x_126, x_30); +lean_inc(x_21); +x_128 = l_Lean_Syntax_node2(x_21, x_28, x_94, x_127); +x_129 = l_Lean_Syntax_node3(x_21, x_14, x_35, x_82, x_128); x_130 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_130, 0, x_129); return x_130; @@ -17140,91 +17140,91 @@ return x_130; 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; x_149 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__0; x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; -lean_inc_ref(x_145); -lean_inc(x_136); -lean_inc(x_142); +lean_inc_ref(x_140); +lean_inc(x_132); +lean_inc(x_138); x_151 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_151, 0, x_142); -lean_ctor_set(x_151, 1, x_136); -lean_ctor_set(x_151, 2, x_145); +lean_ctor_set(x_151, 0, x_138); +lean_ctor_set(x_151, 1, x_132); +lean_ctor_set(x_151, 2, x_140); x_152 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; -lean_inc(x_142); +lean_inc(x_138); x_153 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_153, 0, x_142); +lean_ctor_set(x_153, 0, x_138); lean_ctor_set(x_153, 1, x_152); x_154 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_142); +lean_inc(x_138); x_155 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_155, 0, x_142); +lean_ctor_set(x_155, 0, x_138); lean_ctor_set(x_155, 1, x_154); x_156 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__30; x_157 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__31; -lean_inc(x_132); +lean_inc(x_133); lean_inc(x_147); -x_158 = l_Lean_addMacroScope(x_147, x_157, x_132); +x_158 = l_Lean_addMacroScope(x_147, x_157, x_133); x_159 = lean_box(0); x_160 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__3; -lean_inc(x_137); +lean_inc(x_141); x_161 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_137); -lean_inc(x_142); +lean_ctor_set(x_161, 1, x_141); +lean_inc(x_138); x_162 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_162, 0, x_142); +lean_ctor_set(x_162, 0, x_138); lean_ctor_set(x_162, 1, x_156); lean_ctor_set(x_162, 2, x_158); lean_ctor_set(x_162, 3, x_161); x_163 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_133); -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_164 = l_Lean_Name_mkStr4(x_146, x_138, x_133, x_163); +lean_inc_ref(x_143); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_164 = l_Lean_Name_mkStr4(x_136, x_142, x_143, x_163); x_165 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_133); -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_166 = l_Lean_Name_mkStr4(x_146, x_138, x_133, x_165); +lean_inc_ref(x_143); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_166 = l_Lean_Name_mkStr4(x_136, x_142, x_143, x_165); x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; -lean_inc(x_142); +lean_inc(x_138); x_168 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_168, 0, x_142); +lean_ctor_set(x_168, 0, x_138); lean_ctor_set(x_168, 1, x_167); x_169 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__25; x_170 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__27; x_171 = lean_box(0); -lean_inc(x_132); +lean_inc(x_133); lean_inc(x_147); -x_172 = l_Lean_addMacroScope(x_147, x_171, x_132); +x_172 = l_Lean_addMacroScope(x_147, x_171, x_133); x_173 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__1; x_174 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__59; -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_176 = l_Lean_Name_mkStr3(x_146, x_138, x_175); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_176 = l_Lean_Name_mkStr3(x_136, x_142, x_175); x_177 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_177, 0, x_176); x_178 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_146); -x_179 = l_Lean_Name_mkStr3(x_146, x_178, x_175); +lean_inc_ref(x_136); +x_179 = l_Lean_Name_mkStr3(x_136, x_178, x_175); x_180 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_180, 0, x_179); -lean_inc_ref(x_146); -x_181 = l_Lean_Name_mkStr2(x_146, x_178); +lean_inc_ref(x_136); +x_181 = l_Lean_Name_mkStr2(x_136, x_178); x_182 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_182, 0, x_181); -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_183 = l_Lean_Name_mkStr2(x_146, x_138); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_183 = l_Lean_Name_mkStr2(x_136, x_142); x_184 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_184, 0, x_183); -lean_inc_ref(x_146); -x_185 = l_Lean_Name_mkStr1(x_146); +lean_inc_ref(x_136); +x_185 = l_Lean_Name_mkStr1(x_136); x_186 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_186, 0, x_185); -lean_inc(x_137); +lean_inc(x_141); x_187 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_187, 0, x_186); -lean_ctor_set(x_187, 1, x_137); +lean_ctor_set(x_187, 1, x_141); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_184); lean_ctor_set(x_188, 1, x_187); @@ -17240,95 +17240,95 @@ lean_ctor_set(x_191, 1, x_190); x_192 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_192, 0, x_174); lean_ctor_set(x_192, 1, x_191); -lean_inc(x_142); +lean_inc(x_138); x_193 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_193, 0, x_142); +lean_ctor_set(x_193, 0, x_138); lean_ctor_set(x_193, 1, x_170); lean_ctor_set(x_193, 2, x_172); lean_ctor_set(x_193, 3, x_192); -lean_inc(x_142); -x_194 = l_Lean_Syntax_node1(x_142, x_169, x_193); -lean_inc(x_142); -x_195 = l_Lean_Syntax_node2(x_142, x_166, x_168, x_194); +lean_inc(x_138); +x_194 = l_Lean_Syntax_node1(x_138, x_169, x_193); +lean_inc(x_138); +x_195 = l_Lean_Syntax_node2(x_138, x_166, x_168, x_194); x_196 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__37; x_197 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__38; -lean_inc(x_142); +lean_inc(x_138); x_198 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_198, 0, x_142); +lean_ctor_set(x_198, 0, x_138); lean_ctor_set(x_198, 1, x_197); -lean_inc(x_142); -x_199 = l_Lean_Syntax_node1(x_142, x_196, x_198); +lean_inc(x_138); +x_199 = l_Lean_Syntax_node1(x_138, x_196, x_198); x_200 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__7; -lean_inc(x_142); +lean_inc(x_138); x_201 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_201, 0, x_142); +lean_ctor_set(x_201, 0, x_138); lean_ctor_set(x_201, 1, x_200); -lean_inc(x_141); -lean_inc(x_136); -lean_inc(x_142); -x_202 = l_Lean_Syntax_node1(x_142, x_136, x_141); +lean_inc(x_145); +lean_inc(x_132); +lean_inc(x_138); +x_202 = l_Lean_Syntax_node1(x_138, x_132, x_145); lean_inc(x_199); -lean_inc(x_136); -lean_inc(x_142); -x_203 = l_Lean_Syntax_node3(x_142, x_136, x_199, x_201, x_202); +lean_inc(x_132); +lean_inc(x_138); +x_203 = l_Lean_Syntax_node3(x_138, x_132, x_199, x_201, x_202); x_204 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; -lean_inc(x_142); +lean_inc(x_138); x_205 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_205, 0, x_142); +lean_ctor_set(x_205, 0, x_138); lean_ctor_set(x_205, 1, x_204); -lean_inc(x_142); -x_206 = l_Lean_Syntax_node3(x_142, x_164, x_195, x_203, x_205); +lean_inc(x_138); +x_206 = l_Lean_Syntax_node3(x_138, x_164, x_195, x_203, x_205); x_207 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__14; -lean_inc(x_142); +lean_inc(x_138); x_208 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_208, 0, x_142); +lean_ctor_set(x_208, 0, x_138); lean_ctor_set(x_208, 1, x_207); x_209 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_133); -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_210 = l_Lean_Name_mkStr4(x_146, x_138, x_133, x_209); +lean_inc_ref(x_143); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_210 = l_Lean_Name_mkStr4(x_136, x_142, x_143, x_209); x_211 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_212 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; -lean_inc(x_132); +lean_inc(x_133); lean_inc(x_147); -x_213 = l_Lean_addMacroScope(x_147, x_212, x_132); +x_213 = l_Lean_addMacroScope(x_147, x_212, x_133); x_214 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__8; x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_137); +lean_inc(x_141); x_216 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_137); +lean_ctor_set(x_216, 1, x_141); x_217 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_217, 0, x_214); lean_ctor_set(x_217, 1, x_216); -lean_inc(x_142); +lean_inc(x_138); x_218 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_218, 0, x_142); +lean_ctor_set(x_218, 0, x_138); lean_ctor_set(x_218, 1, x_211); lean_ctor_set(x_218, 2, x_213); lean_ctor_set(x_218, 3, x_217); -lean_inc(x_144); -lean_inc(x_136); -lean_inc(x_142); -x_219 = l_Lean_Syntax_node1(x_142, x_136, x_144); +lean_inc(x_135); +lean_inc(x_132); +lean_inc(x_138); +x_219 = l_Lean_Syntax_node1(x_138, x_132, x_135); lean_inc(x_210); -lean_inc(x_142); -x_220 = l_Lean_Syntax_node2(x_142, x_210, x_218, x_219); +lean_inc(x_138); +x_220 = l_Lean_Syntax_node2(x_138, x_210, x_218, x_219); lean_inc_ref(x_208); lean_inc_ref(x_155); -lean_inc(x_134); +lean_inc(x_146); lean_inc_ref(x_151); -lean_inc(x_142); -x_221 = l_Lean_Syntax_node8(x_142, x_150, x_151, x_153, x_134, x_155, x_162, x_206, x_208, x_220); +lean_inc(x_138); +x_221 = l_Lean_Syntax_node8(x_138, x_150, x_151, x_153, x_146, x_155, x_162, x_206, x_208, x_220); x_222 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_223 = l_Lean_Name_mkStr4(x_146, x_138, x_175, x_222); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_223 = l_Lean_Name_mkStr4(x_136, x_142, x_175, x_222); x_224 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_138); -lean_inc_ref(x_146); -x_225 = l_Lean_Name_mkStr4(x_146, x_138, x_175, x_224); +lean_inc_ref(x_142); +lean_inc_ref(x_136); +x_225 = l_Lean_Name_mkStr4(x_136, x_142, x_175, x_224); if (lean_obj_tag(x_5) == 1) { lean_object* x_226; lean_object* x_227; @@ -17336,36 +17336,36 @@ x_226 = lean_ctor_get(x_5, 0); lean_inc(x_226); lean_dec_ref(x_5); x_227 = l_Array_mkArray1___redArg(x_226); -x_12 = x_134; -x_13 = x_136; -x_14 = x_138; -x_15 = x_223; -x_16 = x_147; -x_17 = x_139; -x_18 = x_175; -x_19 = x_141; -x_20 = x_143; -x_21 = x_144; -x_22 = x_146; -x_23 = x_145; -x_24 = x_173; -x_25 = x_221; +x_12 = x_159; +x_13 = x_208; +x_14 = x_132; +x_15 = x_133; +x_16 = x_155; +x_17 = x_134; +x_18 = x_200; +x_19 = x_225; +x_20 = x_137; +x_21 = x_138; +x_22 = x_139; +x_23 = x_142; +x_24 = x_141; +x_25 = x_199; x_26 = lean_box(0); -x_27 = x_151; -x_28 = x_132; -x_29 = x_133; -x_30 = x_159; -x_31 = x_135; -x_32 = x_137; -x_33 = x_140; -x_34 = x_142; -x_35 = x_208; -x_36 = x_200; -x_37 = x_155; -x_38 = x_149; -x_39 = x_210; -x_40 = x_225; -x_41 = x_199; +x_27 = x_143; +x_28 = x_223; +x_29 = x_145; +x_30 = x_151; +x_31 = x_147; +x_32 = x_173; +x_33 = x_135; +x_34 = x_136; +x_35 = x_221; +x_36 = x_149; +x_37 = x_140; +x_38 = x_210; +x_39 = x_175; +x_40 = x_144; +x_41 = x_146; x_42 = x_227; goto block_131; } @@ -17374,36 +17374,36 @@ else lean_object* x_228; lean_dec(x_5); x_228 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_12 = x_134; -x_13 = x_136; -x_14 = x_138; -x_15 = x_223; -x_16 = x_147; -x_17 = x_139; -x_18 = x_175; -x_19 = x_141; -x_20 = x_143; -x_21 = x_144; -x_22 = x_146; -x_23 = x_145; -x_24 = x_173; -x_25 = x_221; +x_12 = x_159; +x_13 = x_208; +x_14 = x_132; +x_15 = x_133; +x_16 = x_155; +x_17 = x_134; +x_18 = x_200; +x_19 = x_225; +x_20 = x_137; +x_21 = x_138; +x_22 = x_139; +x_23 = x_142; +x_24 = x_141; +x_25 = x_199; x_26 = lean_box(0); -x_27 = x_151; -x_28 = x_132; -x_29 = x_133; -x_30 = x_159; -x_31 = x_135; -x_32 = x_137; -x_33 = x_140; -x_34 = x_142; -x_35 = x_208; -x_36 = x_200; -x_37 = x_155; -x_38 = x_149; -x_39 = x_210; -x_40 = x_225; -x_41 = x_199; +x_27 = x_143; +x_28 = x_223; +x_29 = x_145; +x_30 = x_151; +x_31 = x_147; +x_32 = x_173; +x_33 = x_135; +x_34 = x_136; +x_35 = x_221; +x_36 = x_149; +x_37 = x_140; +x_38 = x_210; +x_39 = x_175; +x_40 = x_144; +x_41 = x_146; x_42 = x_228; goto block_131; } @@ -18188,106 +18188,106 @@ goto block_106; { 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_17 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_15); -lean_inc_ref(x_12); +lean_inc_ref(x_9); lean_inc_ref(x_10); -x_18 = l_Lean_Name_mkStr4(x_10, x_12, x_15, x_17); -x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_15); lean_inc_ref(x_12); +x_18 = l_Lean_Name_mkStr4(x_12, x_10, x_9, x_17); +x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; +lean_inc_ref(x_9); lean_inc_ref(x_10); -x_20 = l_Lean_Name_mkStr4(x_10, x_12, x_15, x_19); +lean_inc_ref(x_12); +x_20 = l_Lean_Name_mkStr4(x_12, x_10, x_9, x_19); x_21 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_22 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_11); +lean_inc(x_14); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_11); +lean_ctor_set(x_23, 0, x_14); lean_ctor_set(x_23, 1, x_21); lean_ctor_set(x_23, 2, x_22); lean_inc_ref_n(x_23, 7); -lean_inc(x_11); -x_24 = l_Lean_Syntax_node7(x_11, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); +lean_inc(x_14); +x_24 = l_Lean_Syntax_node7(x_14, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); x_25 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_15); -lean_inc_ref(x_12); +lean_inc_ref(x_9); lean_inc_ref(x_10); -x_26 = l_Lean_Name_mkStr4(x_10, x_12, x_15, x_25); +lean_inc_ref(x_12); +x_26 = l_Lean_Name_mkStr4(x_12, x_10, x_9, x_25); x_27 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_11); +lean_inc(x_14); x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 0, x_14); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_15); -lean_inc_ref(x_12); +lean_inc_ref(x_9); lean_inc_ref(x_10); -x_30 = l_Lean_Name_mkStr4(x_10, x_12, x_15, x_29); +lean_inc_ref(x_12); +x_30 = l_Lean_Name_mkStr4(x_12, x_10, x_9, x_29); x_31 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; -lean_inc(x_9); +lean_inc(x_8); x_32 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_32, 0, x_9); +lean_ctor_set(x_32, 0, x_8); lean_ctor_set(x_32, 1, x_21); lean_ctor_set(x_32, 2, x_31); x_33 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_34 = lean_array_push(x_33, x_2); x_35 = lean_array_push(x_34, x_32); x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_9); +lean_ctor_set(x_36, 0, x_8); lean_ctor_set(x_36, 1, x_30); lean_ctor_set(x_36, 2, x_35); x_37 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_12); lean_inc_ref(x_10); -x_38 = l_Lean_Name_mkStr4(x_10, x_12, x_15, x_37); +lean_inc_ref(x_12); +x_38 = l_Lean_Name_mkStr4(x_12, x_10, x_9, x_37); x_39 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_40 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -x_41 = l_Lean_Name_mkStr4(x_10, x_12, x_39, x_40); +x_41 = l_Lean_Name_mkStr4(x_12, x_10, x_39, x_40); x_42 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_11); +lean_inc(x_14); x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_11); +lean_ctor_set(x_43, 0, x_14); lean_ctor_set(x_43, 1, x_42); -lean_inc(x_11); -x_44 = l_Lean_Syntax_node2(x_11, x_41, x_43, x_3); -lean_inc(x_11); -x_45 = l_Lean_Syntax_node1(x_11, x_21, x_44); +lean_inc(x_14); +x_44 = l_Lean_Syntax_node2(x_14, x_41, x_43, x_3); +lean_inc(x_14); +x_45 = l_Lean_Syntax_node1(x_14, x_21, x_44); lean_inc_ref(x_23); -lean_inc(x_11); -x_46 = l_Lean_Syntax_node2(x_11, x_38, x_23, x_45); -lean_inc(x_11); -x_47 = l_Lean_Syntax_node5(x_11, x_26, x_28, x_36, x_46, x_13, x_23); -x_48 = l_Lean_Syntax_node2(x_11, x_18, x_24, x_47); +lean_inc(x_14); +x_46 = l_Lean_Syntax_node2(x_14, x_38, x_23, x_45); +lean_inc(x_14); +x_47 = l_Lean_Syntax_node5(x_14, x_26, x_28, x_36, x_46, x_15, x_23); +x_48 = l_Lean_Syntax_node2(x_14, x_18, x_24, x_47); lean_inc(x_48); x_49 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___boxed), 4, 1); lean_closure_set(x_49, 0, x_48); -x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_14, x_8); +x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_11, x_13); return x_50; } block_82: { lean_object* x_62; -x_62 = l_Lean_Elab_Command_getRef___redArg(x_59); +x_62 = l_Lean_Elab_Command_getRef___redArg(x_54); if (lean_obj_tag(x_62) == 0) { lean_object* x_63; lean_object* x_64; x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); lean_dec_ref(x_62); -x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_59); +x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_54); 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; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_dec_ref(x_64); -x_65 = lean_ctor_get(x_59, 5); +x_65 = lean_ctor_get(x_54, 5); x_66 = l_Lean_mkOptionalNode(x_61); x_67 = l_Lake_DSL_elabConfig___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__2___closed__0; -x_68 = lean_array_push(x_67, x_55); +x_68 = lean_array_push(x_67, x_59); x_69 = lean_array_push(x_68, x_58); x_70 = lean_array_push(x_69, x_66); x_71 = lean_box(2); x_72 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_52); +lean_ctor_set(x_72, 1, x_60); lean_ctor_set(x_72, 2, x_70); x_73 = 0; x_74 = l_Lean_SourceInfo_fromRef(x_63, x_73); @@ -18295,29 +18295,29 @@ lean_dec(x_63); if (lean_obj_tag(x_65) == 0) { lean_object* x_75; -x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_54); +x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_57); lean_dec_ref(x_75); -x_8 = x_54; -x_9 = x_71; -x_10 = x_53; -x_11 = x_74; -x_12 = x_57; -x_13 = x_72; -x_14 = x_59; -x_15 = x_60; +x_8 = x_71; +x_9 = x_53; +x_10 = x_52; +x_11 = x_54; +x_12 = x_55; +x_13 = x_57; +x_14 = x_74; +x_15 = x_72; x_16 = lean_box(0); goto block_51; } else { -x_8 = x_54; -x_9 = x_71; -x_10 = x_53; -x_11 = x_74; -x_12 = x_57; -x_13 = x_72; -x_14 = x_59; -x_15 = x_60; +x_8 = x_71; +x_9 = x_53; +x_10 = x_52; +x_11 = x_54; +x_12 = x_55; +x_13 = x_57; +x_14 = x_74; +x_15 = x_72; x_16 = lean_box(0); goto block_51; } @@ -18327,14 +18327,14 @@ else uint8_t x_76; lean_dec(x_63); lean_dec(x_61); -lean_dec_ref(x_60); -lean_dec_ref(x_59); +lean_dec(x_60); +lean_dec(x_59); lean_dec(x_58); -lean_dec_ref(x_57); -lean_dec(x_55); -lean_dec(x_54); +lean_dec(x_57); +lean_dec_ref(x_55); +lean_dec_ref(x_54); lean_dec_ref(x_53); -lean_dec(x_52); +lean_dec_ref(x_52); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -18359,14 +18359,14 @@ else { uint8_t x_79; lean_dec(x_61); -lean_dec_ref(x_60); -lean_dec_ref(x_59); +lean_dec(x_60); +lean_dec(x_59); lean_dec(x_58); -lean_dec_ref(x_57); -lean_dec(x_55); -lean_dec(x_54); +lean_dec(x_57); +lean_dec_ref(x_55); +lean_dec_ref(x_54); lean_dec_ref(x_53); -lean_dec(x_52); +lean_dec_ref(x_52); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -18414,15 +18414,15 @@ if (lean_obj_tag(x_86) == 0) { lean_object* x_99; x_99 = lean_box(0); -x_52 = x_98; -x_53 = x_95; -x_54 = x_88; -x_55 = x_94; +x_52 = x_96; +x_53 = x_97; +x_54 = x_87; +x_55 = x_95; x_56 = lean_box(0); -x_57 = x_96; +x_57 = x_88; x_58 = x_92; -x_59 = x_87; -x_60 = x_97; +x_59 = x_94; +x_60 = x_98; x_61 = x_99; goto block_82; } @@ -18432,15 +18432,15 @@ uint8_t x_100; x_100 = !lean_is_exclusive(x_86); if (x_100 == 0) { -x_52 = x_98; -x_53 = x_95; -x_54 = x_88; -x_55 = x_94; +x_52 = x_96; +x_53 = x_97; +x_54 = x_87; +x_55 = x_95; x_56 = lean_box(0); -x_57 = x_96; +x_57 = x_88; x_58 = x_92; -x_59 = x_87; -x_60 = x_97; +x_59 = x_94; +x_60 = x_98; x_61 = x_86; goto block_82; } @@ -18452,15 +18452,15 @@ lean_inc(x_101); lean_dec(x_86); x_102 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_102, 0, x_101); -x_52 = x_98; -x_53 = x_95; -x_54 = x_88; -x_55 = x_94; +x_52 = x_96; +x_53 = x_97; +x_54 = x_87; +x_55 = x_95; x_56 = lean_box(0); -x_57 = x_96; +x_57 = x_88; x_58 = x_92; -x_59 = x_87; -x_60 = x_97; +x_59 = x_94; +x_60 = x_98; x_61 = x_102; goto block_82; } @@ -18570,22 +18570,22 @@ lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; x_259 = lean_ctor_get(x_258, 0); lean_inc(x_259); lean_dec_ref(x_258); -lean_inc_ref(x_247); -lean_inc(x_236); -lean_inc(x_248); +lean_inc_ref(x_236); +lean_inc(x_244); +lean_inc(x_240); x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_248); -lean_ctor_set(x_260, 1, x_236); -lean_ctor_set(x_260, 2, x_247); +lean_ctor_set(x_260, 0, x_240); +lean_ctor_set(x_260, 1, x_244); +lean_ctor_set(x_260, 2, x_236); lean_inc_ref(x_260); -lean_inc(x_248); -x_261 = l_Lean_Syntax_node1(x_248, x_246, x_260); -lean_inc(x_248); -x_262 = l_Lean_Syntax_node2(x_248, x_242, x_240, x_260); -x_263 = l_Lean_Syntax_node2(x_248, x_238, x_261, x_262); +lean_inc(x_240); +x_261 = l_Lean_Syntax_node1(x_240, x_243, x_260); +lean_inc(x_240); +x_262 = l_Lean_Syntax_node2(x_240, x_246, x_237, x_260); +x_263 = l_Lean_Syntax_node2(x_240, x_245, x_261, x_262); x_264 = lean_unsigned_to_nat(2u); x_265 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -x_266 = lean_array_push(x_265, x_250); +x_266 = lean_array_push(x_265, x_238); x_267 = lean_array_push(x_266, x_263); x_268 = l_Lake_DSL_expandAttrs(x_6); x_269 = l_Array_append___redArg(x_267, x_268); @@ -18600,20 +18600,20 @@ x_272 = lean_ctor_get(x_271, 0); lean_inc(x_272); lean_dec_ref(x_271); x_132 = x_236; -x_133 = x_237; -x_134 = x_259; -x_135 = x_270; -x_136 = x_239; -x_137 = x_241; -x_138 = x_253; -x_139 = x_243; -x_140 = x_244; -x_141 = x_245; -x_142 = x_269; -x_143 = x_247; -x_144 = x_264; +x_133 = x_239; +x_134 = x_241; +x_135 = x_259; +x_136 = x_242; +x_137 = x_269; +x_138 = x_257; +x_139 = x_244; +x_140 = x_270; +x_141 = x_247; +x_142 = x_253; +x_143 = x_248; +x_144 = x_250; x_145 = x_249; -x_146 = x_257; +x_146 = x_264; x_147 = x_272; x_148 = lean_box(0); goto block_229; @@ -18626,20 +18626,20 @@ x_273 = lean_ctor_get(x_234, 0); lean_inc(x_273); lean_dec_ref(x_234); x_132 = x_236; -x_133 = x_237; -x_134 = x_259; -x_135 = x_270; -x_136 = x_239; -x_137 = x_241; -x_138 = x_253; -x_139 = x_243; -x_140 = x_244; -x_141 = x_245; -x_142 = x_269; -x_143 = x_247; -x_144 = x_264; +x_133 = x_239; +x_134 = x_241; +x_135 = x_259; +x_136 = x_242; +x_137 = x_269; +x_138 = x_257; +x_139 = x_244; +x_140 = x_270; +x_141 = x_247; +x_142 = x_253; +x_143 = x_248; +x_144 = x_250; x_145 = x_249; -x_146 = x_257; +x_146 = x_264; x_147 = x_273; x_148 = lean_box(0); goto block_229; @@ -18651,21 +18651,21 @@ uint8_t x_274; lean_dec(x_257); lean_dec(x_255); lean_dec(x_253); -lean_dec(x_250); +lean_dec_ref(x_250); lean_dec_ref(x_249); lean_dec(x_248); lean_dec_ref(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); lean_dec(x_242); -lean_dec_ref(x_241); +lean_dec(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec(x_6); @@ -18693,21 +18693,21 @@ else uint8_t x_277; lean_dec(x_255); lean_dec(x_253); -lean_dec(x_250); +lean_dec_ref(x_250); lean_dec_ref(x_249); lean_dec(x_248); lean_dec_ref(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); lean_dec(x_242); -lean_dec_ref(x_241); +lean_dec(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -18735,21 +18735,21 @@ else { uint8_t x_280; lean_dec(x_253); -lean_dec(x_250); +lean_dec_ref(x_250); lean_dec_ref(x_249); lean_dec(x_248); lean_dec_ref(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); lean_dec(x_242); -lean_dec_ref(x_241); +lean_dec(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -18775,21 +18775,21 @@ return x_282; } else { -lean_dec(x_250); +lean_dec_ref(x_250); lean_dec_ref(x_249); lean_dec(x_248); lean_dec_ref(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); lean_dec(x_242); -lean_dec_ref(x_241); +lean_dec(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -18821,68 +18821,68 @@ x_299 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_300 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_301 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_302 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_286); +lean_inc(x_288); x_303 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_303, 0, x_286); +lean_ctor_set(x_303, 0, x_288); lean_ctor_set(x_303, 1, x_301); lean_ctor_set(x_303, 2, x_302); lean_inc_ref(x_303); -lean_inc(x_286); -x_304 = l_Lean_Syntax_node1(x_286, x_300, x_303); +lean_inc(x_288); +x_304 = l_Lean_Syntax_node1(x_288, x_300, x_303); x_305 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_306 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_307 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_308 = l_Lean_addMacroScope(x_291, x_307, x_290); -lean_inc(x_289); -lean_inc(x_286); +x_308 = l_Lean_addMacroScope(x_291, x_307, x_286); +lean_inc(x_285); +lean_inc(x_288); x_309 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_309, 0, x_286); +lean_ctor_set(x_309, 0, x_288); lean_ctor_set(x_309, 1, x_306); lean_ctor_set(x_309, 2, x_308); -lean_ctor_set(x_309, 3, x_289); -lean_inc(x_286); -x_310 = l_Lean_Syntax_node2(x_286, x_305, x_309, x_303); -x_311 = l_Lean_Syntax_node2(x_286, x_299, x_304, x_310); +lean_ctor_set(x_309, 3, x_285); +lean_inc(x_288); +x_310 = l_Lean_Syntax_node2(x_288, x_305, x_309, x_303); +x_311 = l_Lean_Syntax_node2(x_288, x_299, x_304, x_310); if (lean_obj_tag(x_234) == 0) { lean_object* x_312; x_312 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_10); lean_dec_ref(x_312); -x_236 = x_301; -x_237 = x_285; -x_238 = x_299; -x_239 = x_287; -x_240 = x_288; -x_241 = x_297; -x_242 = x_305; -x_243 = x_289; -x_244 = x_284; -x_245 = x_298; -x_246 = x_300; -x_247 = x_302; -x_248 = x_294; -x_249 = x_296; -x_250 = x_311; +x_236 = x_302; +x_237 = x_284; +x_238 = x_311; +x_239 = x_285; +x_240 = x_294; +x_241 = x_287; +x_242 = x_289; +x_243 = x_300; +x_244 = x_301; +x_245 = x_299; +x_246 = x_305; +x_247 = x_298; +x_248 = x_290; +x_249 = x_297; +x_250 = x_296; x_251 = lean_box(0); goto block_283; } else { -x_236 = x_301; -x_237 = x_285; -x_238 = x_299; -x_239 = x_287; -x_240 = x_288; -x_241 = x_297; -x_242 = x_305; -x_243 = x_289; -x_244 = x_284; -x_245 = x_298; -x_246 = x_300; -x_247 = x_302; -x_248 = x_294; -x_249 = x_296; -x_250 = x_311; +x_236 = x_302; +x_237 = x_284; +x_238 = x_311; +x_239 = x_285; +x_240 = x_294; +x_241 = x_287; +x_242 = x_289; +x_243 = x_300; +x_244 = x_301; +x_245 = x_299; +x_246 = x_305; +x_247 = x_298; +x_248 = x_290; +x_249 = x_297; +x_250 = x_296; x_251 = lean_box(0); goto block_283; } @@ -19022,13 +19022,13 @@ x_342 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkC x_343 = lean_ctor_get(x_342, 0); lean_inc(x_343); lean_dec_ref(x_342); -x_284 = x_324; -x_285 = x_329; -x_286 = x_339; -x_287 = x_331; -x_288 = x_337; -x_289 = x_328; -x_290 = x_341; +x_284 = x_337; +x_285 = x_328; +x_286 = x_341; +x_287 = x_329; +x_288 = x_339; +x_289 = x_324; +x_290 = x_331; x_291 = x_343; x_292 = lean_box(0); goto block_319; @@ -19041,13 +19041,13 @@ lean_inc(x_344); lean_dec_ref(x_340); x_345 = lean_ctor_get(x_234, 0); lean_inc(x_345); -x_284 = x_324; -x_285 = x_329; -x_286 = x_339; -x_287 = x_331; -x_288 = x_337; -x_289 = x_328; -x_290 = x_344; +x_284 = x_337; +x_285 = x_328; +x_286 = x_344; +x_287 = x_329; +x_288 = x_339; +x_289 = x_324; +x_290 = x_331; x_291 = x_345; x_292 = lean_box(0); goto block_319; @@ -19244,43 +19244,43 @@ return x_364; block_131: { 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_inc_ref(x_19); -x_43 = l_Array_append___redArg(x_19, x_42); +lean_inc_ref(x_28); +x_43 = l_Array_append___redArg(x_28, x_42); lean_dec_ref(x_42); -lean_inc(x_22); -lean_inc(x_21); +lean_inc(x_35); +lean_inc(x_36); x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_21); -lean_ctor_set(x_44, 1, x_22); +lean_ctor_set(x_44, 0, x_36); +lean_ctor_set(x_44, 1, x_35); lean_ctor_set(x_44, 2, x_43); -lean_inc_n(x_15, 6); -lean_inc(x_23); -lean_inc(x_21); -x_45 = l_Lean_Syntax_node7(x_21, x_23, x_44, x_15, x_15, x_15, x_15, x_15, x_15); +lean_inc_n(x_41, 6); +lean_inc(x_33); +lean_inc(x_36); +x_45 = l_Lean_Syntax_node7(x_36, x_33, x_44, x_41, x_41, x_41, x_41, x_41, x_41); x_46 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_41); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_47 = l_Lean_Name_mkStr4(x_20, x_30, x_41, x_46); -lean_inc(x_21); +lean_inc_ref(x_21); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_47 = l_Lean_Name_mkStr4(x_39, x_26, x_21, x_46); +lean_inc(x_36); x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_21); +lean_ctor_set(x_48, 0, x_36); lean_ctor_set(x_48, 1, x_46); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_41); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_50 = l_Lean_Name_mkStr4(x_20, x_30, x_41, x_49); +lean_inc_ref(x_21); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_50 = l_Lean_Name_mkStr4(x_39, x_26, x_21, x_49); x_51 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_52 = lean_box(2); -lean_inc(x_22); +lean_inc(x_35); x_53 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_22); +lean_ctor_set(x_53, 1, x_35); lean_ctor_set(x_53, 2, x_51); -x_54 = lean_mk_empty_array_with_capacity(x_37); -lean_inc(x_33); -x_55 = lean_array_push(x_54, x_33); +x_54 = lean_mk_empty_array_with_capacity(x_40); +lean_inc(x_14); +x_55 = lean_array_push(x_54, x_14); x_56 = lean_array_push(x_55, x_53); lean_inc(x_50); x_57 = lean_alloc_ctor(1, 3, 0); @@ -19288,194 +19288,194 @@ lean_ctor_set(x_57, 0, x_52); lean_ctor_set(x_57, 1, x_50); lean_ctor_set(x_57, 2, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_41); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_59 = l_Lean_Name_mkStr4(x_20, x_30, x_41, x_58); +lean_inc_ref(x_21); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_59 = l_Lean_Name_mkStr4(x_39, x_26, x_21, x_58); x_60 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_34); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_61 = l_Lean_Name_mkStr4(x_20, x_30, x_34, x_60); -lean_inc(x_18); +lean_inc_ref(x_24); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_61 = l_Lean_Name_mkStr4(x_39, x_26, x_24, x_60); +lean_inc(x_30); lean_inc(x_61); -lean_inc(x_21); -x_62 = l_Lean_Syntax_node2(x_21, x_61, x_18, x_29); -lean_inc(x_22); -lean_inc(x_21); -x_63 = l_Lean_Syntax_node1(x_21, x_22, x_62); -lean_inc(x_15); +lean_inc(x_36); +x_62 = l_Lean_Syntax_node2(x_36, x_61, x_30, x_23); +lean_inc(x_35); +lean_inc(x_36); +x_63 = l_Lean_Syntax_node1(x_36, x_35, x_62); +lean_inc(x_41); lean_inc(x_59); -lean_inc(x_21); -x_64 = l_Lean_Syntax_node2(x_21, x_59, x_15, x_63); +lean_inc(x_36); +x_64 = l_Lean_Syntax_node2(x_36, x_59, x_41, x_63); x_65 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__60; -lean_inc_ref(x_41); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_66 = l_Lean_Name_mkStr4(x_20, x_30, x_41, x_65); +lean_inc_ref(x_21); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_66 = l_Lean_Name_mkStr4(x_39, x_26, x_21, x_65); x_67 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__1; x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__2; -lean_inc_ref(x_24); -x_69 = l_Lean_Name_mkStr3(x_24, x_25, x_68); +lean_inc_ref(x_12); +x_69 = l_Lean_Name_mkStr3(x_12, x_17, x_68); lean_inc(x_13); lean_inc(x_69); -lean_inc(x_31); -x_70 = l_Lean_addMacroScope(x_31, x_69, x_13); -lean_inc(x_36); +lean_inc(x_37); +x_70 = l_Lean_addMacroScope(x_37, x_69, x_13); +lean_inc(x_18); x_71 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_36); -lean_inc(x_17); +lean_ctor_set(x_71, 1, x_18); +lean_inc(x_29); x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_17); -lean_inc(x_21); +lean_ctor_set(x_72, 1, x_29); +lean_inc(x_36); x_73 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_73, 0, x_21); +lean_ctor_set(x_73, 0, x_36); lean_ctor_set(x_73, 1, x_67); lean_ctor_set(x_73, 2, x_70); lean_ctor_set(x_73, 3, x_72); -lean_inc(x_22); -lean_inc(x_21); -x_74 = l_Lean_Syntax_node4(x_21, x_22, x_40, x_28, x_26, x_12); -lean_inc(x_21); -x_75 = l_Lean_Syntax_node2(x_21, x_38, x_73, x_74); +lean_inc(x_35); +lean_inc(x_36); +x_74 = l_Lean_Syntax_node4(x_36, x_35, x_27, x_25, x_22, x_31); +lean_inc(x_36); +x_75 = l_Lean_Syntax_node2(x_36, x_16, x_73, x_74); x_76 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__62; x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__63; -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_78 = l_Lean_Name_mkStr4(x_20, x_30, x_76, x_77); -lean_inc_n(x_15, 2); -lean_inc(x_21); -x_79 = l_Lean_Syntax_node2(x_21, x_78, x_15, x_15); -lean_inc(x_15); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_78 = l_Lean_Name_mkStr4(x_39, x_26, x_76, x_77); +lean_inc_n(x_41, 2); +lean_inc(x_36); +x_79 = l_Lean_Syntax_node2(x_36, x_78, x_41, x_41); +lean_inc(x_41); lean_inc(x_79); -lean_inc(x_16); +lean_inc(x_20); lean_inc(x_66); -lean_inc(x_21); -x_80 = l_Lean_Syntax_node4(x_21, x_66, x_16, x_75, x_79, x_15); -lean_inc(x_21); -x_81 = l_Lean_Syntax_node4(x_21, x_47, x_48, x_57, x_64, x_80); -lean_inc(x_32); -lean_inc(x_21); -x_82 = l_Lean_Syntax_node2(x_21, x_32, x_45, x_81); +lean_inc(x_36); +x_80 = l_Lean_Syntax_node4(x_36, x_66, x_20, x_75, x_79, x_41); +lean_inc(x_36); +x_81 = l_Lean_Syntax_node4(x_36, x_47, x_48, x_57, x_64, x_80); +lean_inc(x_38); +lean_inc(x_36); +x_82 = l_Lean_Syntax_node2(x_36, x_38, x_45, x_81); x_83 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_34); -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_84 = l_Lean_Name_mkStr4(x_20, x_30, x_34, x_83); +lean_inc_ref(x_24); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_84 = l_Lean_Name_mkStr4(x_39, x_26, x_24, x_83); x_85 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_21); +lean_inc(x_36); x_86 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_86, 0, x_21); +lean_ctor_set(x_86, 0, x_36); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Syntax_SepArray_ofElems(x_27, x_35); -lean_dec_ref(x_35); -x_88 = l_Array_append___redArg(x_19, x_87); +x_87 = l_Lean_Syntax_SepArray_ofElems(x_19, x_15); +lean_dec_ref(x_15); +x_88 = l_Array_append___redArg(x_28, x_87); lean_dec_ref(x_87); -lean_inc(x_22); -lean_inc(x_21); +lean_inc(x_35); +lean_inc(x_36); x_89 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_89, 0, x_21); -lean_ctor_set(x_89, 1, x_22); +lean_ctor_set(x_89, 0, x_36); +lean_ctor_set(x_89, 1, x_35); lean_ctor_set(x_89, 2, x_88); x_90 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_21); +lean_inc(x_36); x_91 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_91, 0, x_21); +lean_ctor_set(x_91, 0, x_36); lean_ctor_set(x_91, 1, x_90); -lean_inc(x_21); -x_92 = l_Lean_Syntax_node3(x_21, x_84, x_86, x_89, x_91); -lean_inc(x_22); -lean_inc(x_21); -x_93 = l_Lean_Syntax_node1(x_21, x_22, x_92); -lean_inc_n(x_15, 6); -lean_inc(x_21); -x_94 = l_Lean_Syntax_node7(x_21, x_23, x_15, x_93, x_15, x_15, x_15, x_15, x_15); +lean_inc(x_36); +x_92 = l_Lean_Syntax_node3(x_36, x_84, x_86, x_89, x_91); +lean_inc(x_35); +lean_inc(x_36); +x_93 = l_Lean_Syntax_node1(x_36, x_35, x_92); +lean_inc_n(x_41, 6); +lean_inc(x_36); +x_94 = l_Lean_Syntax_node7(x_36, x_33, x_41, x_93, x_41, x_41, x_41, x_41, x_41); x_95 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_30); -lean_inc_ref(x_20); -x_96 = l_Lean_Name_mkStr4(x_20, x_30, x_41, x_95); +lean_inc_ref(x_26); +lean_inc_ref(x_39); +x_96 = l_Lean_Name_mkStr4(x_39, x_26, x_21, x_95); x_97 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_21); +lean_inc(x_36); x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_21); +lean_ctor_set(x_98, 0, x_36); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_100 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; lean_inc(x_13); -lean_inc(x_31); -x_101 = l_Lean_addMacroScope(x_31, x_100, x_13); -lean_inc(x_17); -lean_inc(x_21); +lean_inc(x_37); +x_101 = l_Lean_addMacroScope(x_37, x_100, x_13); +lean_inc(x_29); +lean_inc(x_36); x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_21); +lean_ctor_set(x_102, 0, x_36); lean_ctor_set(x_102, 1, x_99); lean_ctor_set(x_102, 2, x_101); -lean_ctor_set(x_102, 3, x_17); -lean_inc(x_15); -lean_inc(x_21); -x_103 = l_Lean_Syntax_node2(x_21, x_50, x_102, x_15); +lean_ctor_set(x_102, 3, x_29); +lean_inc(x_41); +lean_inc(x_36); +x_103 = l_Lean_Syntax_node2(x_36, x_50, x_102, x_41); x_104 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__5; x_105 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_106 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; lean_inc(x_13); -lean_inc(x_31); -x_107 = l_Lean_addMacroScope(x_31, x_106, x_13); -x_108 = l_Lean_Name_mkStr2(x_24, x_104); +lean_inc(x_37); +x_107 = l_Lean_addMacroScope(x_37, x_106, x_13); +x_108 = l_Lean_Name_mkStr2(x_12, x_104); lean_inc(x_108); x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_36); +lean_ctor_set(x_109, 1, x_18); x_110 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_110, 0, x_108); -lean_inc(x_17); +lean_inc(x_29); x_111 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_17); +lean_ctor_set(x_111, 1, x_29); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_109); lean_ctor_set(x_112, 1, x_111); -lean_inc(x_21); +lean_inc(x_36); x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_21); +lean_ctor_set(x_113, 0, x_36); lean_ctor_set(x_113, 1, x_105); lean_ctor_set(x_113, 2, x_107); lean_ctor_set(x_113, 3, x_112); -lean_inc(x_21); -x_114 = l_Lean_Syntax_node2(x_21, x_61, x_18, x_113); -lean_inc(x_22); -lean_inc(x_21); -x_115 = l_Lean_Syntax_node1(x_21, x_22, x_114); -lean_inc(x_15); -lean_inc(x_21); -x_116 = l_Lean_Syntax_node2(x_21, x_59, x_15, x_115); +lean_inc(x_36); +x_114 = l_Lean_Syntax_node2(x_36, x_61, x_30, x_113); +lean_inc(x_35); +lean_inc(x_36); +x_115 = l_Lean_Syntax_node1(x_36, x_35, x_114); +lean_inc(x_41); +lean_inc(x_36); +x_116 = l_Lean_Syntax_node2(x_36, x_59, x_41, x_115); x_117 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_118 = l_Lean_Name_mkStr4(x_20, x_30, x_34, x_117); +x_118 = l_Lean_Name_mkStr4(x_39, x_26, x_24, x_117); x_119 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_21); +lean_inc(x_36); x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_21); +lean_ctor_set(x_120, 0, x_36); lean_ctor_set(x_120, 1, x_119); x_121 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_122 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_123 = l_Lean_addMacroScope(x_31, x_122, x_13); -lean_inc(x_21); +x_123 = l_Lean_addMacroScope(x_37, x_122, x_13); +lean_inc(x_36); x_124 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_124, 0, x_21); +lean_ctor_set(x_124, 0, x_36); lean_ctor_set(x_124, 1, x_121); lean_ctor_set(x_124, 2, x_123); -lean_ctor_set(x_124, 3, x_17); -lean_inc(x_21); -x_125 = l_Lean_Syntax_node3(x_21, x_118, x_33, x_120, x_124); -lean_inc(x_15); -lean_inc(x_21); -x_126 = l_Lean_Syntax_node4(x_21, x_66, x_16, x_125, x_79, x_15); -lean_inc(x_21); -x_127 = l_Lean_Syntax_node5(x_21, x_96, x_98, x_103, x_116, x_126, x_15); -lean_inc(x_21); -x_128 = l_Lean_Syntax_node2(x_21, x_32, x_94, x_127); -x_129 = l_Lean_Syntax_node3(x_21, x_22, x_39, x_82, x_128); +lean_ctor_set(x_124, 3, x_29); +lean_inc(x_36); +x_125 = l_Lean_Syntax_node3(x_36, x_118, x_14, x_120, x_124); +lean_inc(x_41); +lean_inc(x_36); +x_126 = l_Lean_Syntax_node4(x_36, x_66, x_20, x_125, x_79, x_41); +lean_inc(x_36); +x_127 = l_Lean_Syntax_node5(x_36, x_96, x_98, x_103, x_116, x_126, x_41); +lean_inc(x_36); +x_128 = l_Lean_Syntax_node2(x_36, x_38, x_94, x_127); +x_129 = l_Lean_Syntax_node3(x_36, x_35, x_34, x_82, x_128); x_130 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_130, 0, x_129); return x_130; @@ -19485,91 +19485,91 @@ return x_130; 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; x_149 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__0; x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; -lean_inc_ref(x_143); -lean_inc(x_132); -lean_inc(x_146); +lean_inc_ref(x_132); +lean_inc(x_139); +lean_inc(x_138); x_151 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_151, 0, x_146); -lean_ctor_set(x_151, 1, x_132); -lean_ctor_set(x_151, 2, x_143); +lean_ctor_set(x_151, 0, x_138); +lean_ctor_set(x_151, 1, x_139); +lean_ctor_set(x_151, 2, x_132); x_152 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; -lean_inc(x_146); +lean_inc(x_138); x_153 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_153, 0, x_146); +lean_ctor_set(x_153, 0, x_138); lean_ctor_set(x_153, 1, x_152); x_154 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_146); +lean_inc(x_138); x_155 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_155, 0, x_146); +lean_ctor_set(x_155, 0, x_138); lean_ctor_set(x_155, 1, x_154); x_156 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__30; x_157 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__31; -lean_inc(x_134); +lean_inc(x_135); lean_inc(x_147); -x_158 = l_Lean_addMacroScope(x_147, x_157, x_134); +x_158 = l_Lean_addMacroScope(x_147, x_157, x_135); x_159 = lean_box(0); x_160 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__3; -lean_inc(x_139); +lean_inc(x_133); x_161 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_139); -lean_inc(x_146); +lean_ctor_set(x_161, 1, x_133); +lean_inc(x_138); x_162 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_162, 0, x_146); +lean_ctor_set(x_162, 0, x_138); lean_ctor_set(x_162, 1, x_156); lean_ctor_set(x_162, 2, x_158); lean_ctor_set(x_162, 3, x_161); x_163 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; lean_inc_ref(x_141); -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_164 = l_Lean_Name_mkStr4(x_145, x_137, x_141, x_163); +lean_inc_ref(x_144); +x_164 = l_Lean_Name_mkStr4(x_144, x_145, x_141, x_163); x_165 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; lean_inc_ref(x_141); -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_166 = l_Lean_Name_mkStr4(x_145, x_137, x_141, x_165); +lean_inc_ref(x_144); +x_166 = l_Lean_Name_mkStr4(x_144, x_145, x_141, x_165); x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; -lean_inc(x_146); +lean_inc(x_138); x_168 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_168, 0, x_146); +lean_ctor_set(x_168, 0, x_138); lean_ctor_set(x_168, 1, x_167); x_169 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__25; x_170 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__27; x_171 = lean_box(0); -lean_inc(x_134); +lean_inc(x_135); lean_inc(x_147); -x_172 = l_Lean_addMacroScope(x_147, x_171, x_134); +x_172 = l_Lean_addMacroScope(x_147, x_171, x_135); x_173 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__1; x_174 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__59; -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_176 = l_Lean_Name_mkStr3(x_145, x_137, x_175); +lean_inc_ref(x_144); +x_176 = l_Lean_Name_mkStr3(x_144, x_145, x_175); x_177 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_177, 0, x_176); x_178 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_145); -x_179 = l_Lean_Name_mkStr3(x_145, x_178, x_175); +lean_inc_ref(x_144); +x_179 = l_Lean_Name_mkStr3(x_144, x_178, x_175); x_180 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_180, 0, x_179); -lean_inc_ref(x_145); -x_181 = l_Lean_Name_mkStr2(x_145, x_178); +lean_inc_ref(x_144); +x_181 = l_Lean_Name_mkStr2(x_144, x_178); x_182 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_182, 0, x_181); -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_183 = l_Lean_Name_mkStr2(x_145, x_137); +lean_inc_ref(x_144); +x_183 = l_Lean_Name_mkStr2(x_144, x_145); x_184 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_184, 0, x_183); -lean_inc_ref(x_145); -x_185 = l_Lean_Name_mkStr1(x_145); +lean_inc_ref(x_144); +x_185 = l_Lean_Name_mkStr1(x_144); x_186 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_186, 0, x_185); -lean_inc(x_139); +lean_inc(x_133); x_187 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_187, 0, x_186); -lean_ctor_set(x_187, 1, x_139); +lean_ctor_set(x_187, 1, x_133); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_184); lean_ctor_set(x_188, 1, x_187); @@ -19585,95 +19585,95 @@ lean_ctor_set(x_191, 1, x_190); x_192 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_192, 0, x_174); lean_ctor_set(x_192, 1, x_191); -lean_inc(x_146); +lean_inc(x_138); x_193 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_193, 0, x_146); +lean_ctor_set(x_193, 0, x_138); lean_ctor_set(x_193, 1, x_170); lean_ctor_set(x_193, 2, x_172); lean_ctor_set(x_193, 3, x_192); -lean_inc(x_146); -x_194 = l_Lean_Syntax_node1(x_146, x_169, x_193); -lean_inc(x_146); -x_195 = l_Lean_Syntax_node2(x_146, x_166, x_168, x_194); +lean_inc(x_138); +x_194 = l_Lean_Syntax_node1(x_138, x_169, x_193); +lean_inc(x_138); +x_195 = l_Lean_Syntax_node2(x_138, x_166, x_168, x_194); x_196 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__37; x_197 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__38; -lean_inc(x_146); +lean_inc(x_138); x_198 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_198, 0, x_146); +lean_ctor_set(x_198, 0, x_138); lean_ctor_set(x_198, 1, x_197); -lean_inc(x_146); -x_199 = l_Lean_Syntax_node1(x_146, x_196, x_198); +lean_inc(x_138); +x_199 = l_Lean_Syntax_node1(x_138, x_196, x_198); x_200 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__7; -lean_inc(x_146); +lean_inc(x_138); x_201 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_201, 0, x_146); +lean_ctor_set(x_201, 0, x_138); lean_ctor_set(x_201, 1, x_200); -lean_inc(x_136); -lean_inc(x_132); -lean_inc(x_146); -x_202 = l_Lean_Syntax_node1(x_146, x_132, x_136); +lean_inc(x_143); +lean_inc(x_139); +lean_inc(x_138); +x_202 = l_Lean_Syntax_node1(x_138, x_139, x_143); lean_inc(x_199); -lean_inc(x_132); -lean_inc(x_146); -x_203 = l_Lean_Syntax_node3(x_146, x_132, x_199, x_201, x_202); +lean_inc(x_139); +lean_inc(x_138); +x_203 = l_Lean_Syntax_node3(x_138, x_139, x_199, x_201, x_202); x_204 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; -lean_inc(x_146); +lean_inc(x_138); x_205 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_205, 0, x_146); +lean_ctor_set(x_205, 0, x_138); lean_ctor_set(x_205, 1, x_204); -lean_inc(x_146); -x_206 = l_Lean_Syntax_node3(x_146, x_164, x_195, x_203, x_205); +lean_inc(x_138); +x_206 = l_Lean_Syntax_node3(x_138, x_164, x_195, x_203, x_205); x_207 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__14; -lean_inc(x_146); +lean_inc(x_138); x_208 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_208, 0, x_146); +lean_ctor_set(x_208, 0, x_138); lean_ctor_set(x_208, 1, x_207); x_209 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; lean_inc_ref(x_141); -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_210 = l_Lean_Name_mkStr4(x_145, x_137, x_141, x_209); +lean_inc_ref(x_144); +x_210 = l_Lean_Name_mkStr4(x_144, x_145, x_141, x_209); x_211 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_212 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; -lean_inc(x_134); +lean_inc(x_135); lean_inc(x_147); -x_213 = l_Lean_addMacroScope(x_147, x_212, x_134); +x_213 = l_Lean_addMacroScope(x_147, x_212, x_135); x_214 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__8; x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_139); +lean_inc(x_133); x_216 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_139); +lean_ctor_set(x_216, 1, x_133); x_217 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_217, 0, x_214); lean_ctor_set(x_217, 1, x_216); -lean_inc(x_146); +lean_inc(x_138); x_218 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_218, 0, x_146); +lean_ctor_set(x_218, 0, x_138); lean_ctor_set(x_218, 1, x_211); lean_ctor_set(x_218, 2, x_213); lean_ctor_set(x_218, 3, x_217); -lean_inc(x_135); -lean_inc(x_132); -lean_inc(x_146); -x_219 = l_Lean_Syntax_node1(x_146, x_132, x_135); +lean_inc(x_140); +lean_inc(x_139); +lean_inc(x_138); +x_219 = l_Lean_Syntax_node1(x_138, x_139, x_140); lean_inc(x_210); -lean_inc(x_146); -x_220 = l_Lean_Syntax_node2(x_146, x_210, x_218, x_219); +lean_inc(x_138); +x_220 = l_Lean_Syntax_node2(x_138, x_210, x_218, x_219); lean_inc_ref(x_208); lean_inc_ref(x_155); -lean_inc(x_140); +lean_inc(x_136); lean_inc_ref(x_151); -lean_inc(x_146); -x_221 = l_Lean_Syntax_node8(x_146, x_150, x_151, x_153, x_140, x_155, x_162, x_206, x_208, x_220); +lean_inc(x_138); +x_221 = l_Lean_Syntax_node8(x_138, x_150, x_151, x_153, x_136, x_155, x_162, x_206, x_208, x_220); x_222 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_223 = l_Lean_Name_mkStr4(x_145, x_137, x_175, x_222); +lean_inc_ref(x_144); +x_223 = l_Lean_Name_mkStr4(x_144, x_145, x_175, x_222); x_224 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_137); lean_inc_ref(x_145); -x_225 = l_Lean_Name_mkStr4(x_145, x_137, x_175, x_224); +lean_inc_ref(x_144); +x_225 = l_Lean_Name_mkStr4(x_144, x_145, x_175, x_224); if (lean_obj_tag(x_5) == 1) { lean_object* x_226; lean_object* x_227; @@ -19681,36 +19681,36 @@ x_226 = lean_ctor_get(x_5, 0); lean_inc(x_226); lean_dec_ref(x_5); x_227 = l_Array_mkArray1___redArg(x_226); -x_12 = x_133; -x_13 = x_134; -x_14 = lean_box(0); -x_15 = x_151; -x_16 = x_208; -x_17 = x_139; -x_18 = x_155; -x_19 = x_143; -x_20 = x_145; -x_21 = x_146; -x_22 = x_132; -x_23 = x_225; -x_24 = x_149; -x_25 = x_173; -x_26 = x_135; -x_27 = x_200; -x_28 = x_136; -x_29 = x_138; -x_30 = x_137; -x_31 = x_147; -x_32 = x_223; -x_33 = x_140; -x_34 = x_141; -x_35 = x_142; -x_36 = x_159; -x_37 = x_144; -x_38 = x_210; -x_39 = x_221; -x_40 = x_199; -x_41 = x_175; +x_12 = x_149; +x_13 = x_135; +x_14 = x_136; +x_15 = x_137; +x_16 = x_210; +x_17 = x_173; +x_18 = x_159; +x_19 = x_200; +x_20 = x_208; +x_21 = x_175; +x_22 = x_140; +x_23 = x_142; +x_24 = x_141; +x_25 = x_143; +x_26 = x_145; +x_27 = x_199; +x_28 = x_132; +x_29 = x_133; +x_30 = x_155; +x_31 = x_134; +x_32 = lean_box(0); +x_33 = x_225; +x_34 = x_221; +x_35 = x_139; +x_36 = x_138; +x_37 = x_147; +x_38 = x_223; +x_39 = x_144; +x_40 = x_146; +x_41 = x_151; x_42 = x_227; goto block_131; } @@ -19719,36 +19719,36 @@ else lean_object* x_228; lean_dec(x_5); x_228 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_12 = x_133; -x_13 = x_134; -x_14 = lean_box(0); -x_15 = x_151; -x_16 = x_208; -x_17 = x_139; -x_18 = x_155; -x_19 = x_143; -x_20 = x_145; -x_21 = x_146; -x_22 = x_132; -x_23 = x_225; -x_24 = x_149; -x_25 = x_173; -x_26 = x_135; -x_27 = x_200; -x_28 = x_136; -x_29 = x_138; -x_30 = x_137; -x_31 = x_147; -x_32 = x_223; -x_33 = x_140; -x_34 = x_141; -x_35 = x_142; -x_36 = x_159; -x_37 = x_144; -x_38 = x_210; -x_39 = x_221; -x_40 = x_199; -x_41 = x_175; +x_12 = x_149; +x_13 = x_135; +x_14 = x_136; +x_15 = x_137; +x_16 = x_210; +x_17 = x_173; +x_18 = x_159; +x_19 = x_200; +x_20 = x_208; +x_21 = x_175; +x_22 = x_140; +x_23 = x_142; +x_24 = x_141; +x_25 = x_143; +x_26 = x_145; +x_27 = x_199; +x_28 = x_132; +x_29 = x_133; +x_30 = x_155; +x_31 = x_134; +x_32 = lean_box(0); +x_33 = x_225; +x_34 = x_221; +x_35 = x_139; +x_36 = x_138; +x_37 = x_147; +x_38 = x_223; +x_39 = x_144; +x_40 = x_146; +x_41 = x_151; x_42 = x_228; goto block_131; } @@ -19839,7 +19839,7 @@ lean_dec(x_14); lean_ctor_set(x_2, 7, x_29); lean_inc(x_3); lean_inc_ref(x_2); -x_30 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputfileCommand_spec__0(x_27, x_28, x_28, x_26, x_21, x_19, x_20, x_18, x_2, x_3); +x_30 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputfileCommand_spec__0(x_27, x_28, x_28, x_26, x_21, x_20, x_19, x_18, x_2, x_3); if (lean_obj_tag(x_30) == 0) { lean_object* x_31; lean_object* x_32; lean_object* x_33; @@ -19918,7 +19918,7 @@ lean_ctor_set(x_51, 9, x_45); lean_ctor_set_uint8(x_51, sizeof(void*)*10, x_46); lean_inc(x_3); lean_inc_ref(x_51); -x_52 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputfileCommand_spec__0(x_48, x_49, x_49, x_47, x_21, x_19, x_20, x_18, x_51, x_3); +x_52 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputfileCommand_spec__0(x_48, x_49, x_49, x_47, x_21, x_20, x_19, x_18, x_51, x_3); if (lean_obj_tag(x_52) == 0) { lean_object* x_53; lean_object* x_54; lean_object* x_55; @@ -19993,8 +19993,8 @@ if (lean_obj_tag(x_65) == 0) { lean_object* x_66; x_66 = lean_box(0); -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_66; goto block_62; } @@ -20004,8 +20004,8 @@ uint8_t x_67; x_67 = !lean_is_exclusive(x_65); if (x_67 == 0) { -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_65; goto block_62; } @@ -20017,8 +20017,8 @@ lean_inc(x_68); lean_dec(x_65); x_69 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_69, 0, x_68); -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_69; goto block_62; } @@ -20533,101 +20533,101 @@ goto block_106; { 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_17 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_13); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_9); -x_18 = l_Lean_Name_mkStr4(x_9, x_11, x_13, x_17); +x_18 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_17); x_19 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_13); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_9); -x_20 = l_Lean_Name_mkStr4(x_9, x_11, x_13, x_19); +x_20 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_19); x_21 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_22 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_10); +lean_inc(x_8); x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_10); +lean_ctor_set(x_23, 0, x_8); lean_ctor_set(x_23, 1, x_21); lean_ctor_set(x_23, 2, x_22); lean_inc_ref_n(x_23, 7); -lean_inc(x_10); -x_24 = l_Lean_Syntax_node7(x_10, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); +lean_inc(x_8); +x_24 = l_Lean_Syntax_node7(x_8, x_20, x_23, x_23, x_23, x_23, x_23, x_23, x_23); x_25 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_13); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_9); -x_26 = l_Lean_Name_mkStr4(x_9, x_11, x_13, x_25); +x_26 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_25); x_27 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_10); +lean_inc(x_8); x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_10); +lean_ctor_set(x_28, 0, x_8); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_13); +lean_inc_ref(x_10); +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_9); -x_30 = l_Lean_Name_mkStr4(x_9, x_11, x_13, x_29); +x_30 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_29); x_31 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; -lean_inc(x_15); +lean_inc(x_13); x_32 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_32, 0, x_15); +lean_ctor_set(x_32, 0, x_13); lean_ctor_set(x_32, 1, x_21); lean_ctor_set(x_32, 2, x_31); x_33 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_34 = lean_array_push(x_33, x_2); x_35 = lean_array_push(x_34, x_32); x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_15); +lean_ctor_set(x_36, 0, x_13); lean_ctor_set(x_36, 1, x_30); lean_ctor_set(x_36, 2, x_35); x_37 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; +lean_inc_ref(x_15); lean_inc_ref(x_11); -lean_inc_ref(x_9); -x_38 = l_Lean_Name_mkStr4(x_9, x_11, x_13, x_37); +x_38 = l_Lean_Name_mkStr4(x_11, x_15, x_10, x_37); x_39 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_40 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -x_41 = l_Lean_Name_mkStr4(x_9, x_11, x_39, x_40); +x_41 = l_Lean_Name_mkStr4(x_11, x_15, x_39, x_40); x_42 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_10); +lean_inc(x_8); x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_10); +lean_ctor_set(x_43, 0, x_8); lean_ctor_set(x_43, 1, x_42); -lean_inc(x_10); -x_44 = l_Lean_Syntax_node2(x_10, x_41, x_43, x_3); -lean_inc(x_10); -x_45 = l_Lean_Syntax_node1(x_10, x_21, x_44); +lean_inc(x_8); +x_44 = l_Lean_Syntax_node2(x_8, x_41, x_43, x_3); +lean_inc(x_8); +x_45 = l_Lean_Syntax_node1(x_8, x_21, x_44); lean_inc_ref(x_23); -lean_inc(x_10); -x_46 = l_Lean_Syntax_node2(x_10, x_38, x_23, x_45); -lean_inc(x_10); -x_47 = l_Lean_Syntax_node5(x_10, x_26, x_28, x_36, x_46, x_8, x_23); -x_48 = l_Lean_Syntax_node2(x_10, x_18, x_24, x_47); +lean_inc(x_8); +x_46 = l_Lean_Syntax_node2(x_8, x_38, x_23, x_45); +lean_inc(x_8); +x_47 = l_Lean_Syntax_node5(x_8, x_26, x_28, x_36, x_46, x_14, x_23); +x_48 = l_Lean_Syntax_node2(x_8, x_18, x_24, x_47); lean_inc(x_48); x_49 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___boxed), 4, 1); lean_closure_set(x_49, 0, x_48); -x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_12, x_14); +x_50 = l_Lean_Elab_Command_withMacroExpansion___redArg(x_4, x_48, x_49, x_9, x_12); return x_50; } block_82: { lean_object* x_62; -x_62 = l_Lean_Elab_Command_getRef___redArg(x_57); +x_62 = l_Lean_Elab_Command_getRef___redArg(x_53); if (lean_obj_tag(x_62) == 0) { lean_object* x_63; lean_object* x_64; x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); lean_dec_ref(x_62); -x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_57); +x_64 = l_Lean_Elab_Command_getCurrMacroScope___redArg(x_53); 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; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_dec_ref(x_64); -x_65 = lean_ctor_get(x_57, 5); +x_65 = lean_ctor_get(x_53, 5); x_66 = l_Lean_mkOptionalNode(x_61); x_67 = l_Lake_DSL_elabConfig___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__2___closed__0; -x_68 = lean_array_push(x_67, x_60); -x_69 = lean_array_push(x_68, x_56); +x_68 = lean_array_push(x_67, x_55); +x_69 = lean_array_push(x_68, x_54); x_70 = lean_array_push(x_69, x_66); x_71 = lean_box(2); x_72 = lean_alloc_ctor(1, 3, 0); @@ -20642,27 +20642,27 @@ if (lean_obj_tag(x_65) == 0) lean_object* x_75; x_75 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_58); lean_dec_ref(x_75); -x_8 = x_72; +x_8 = x_74; x_9 = x_53; -x_10 = x_74; -x_11 = x_54; -x_12 = x_57; -x_13 = x_55; -x_14 = x_58; -x_15 = x_71; +x_10 = x_57; +x_11 = x_56; +x_12 = x_58; +x_13 = x_71; +x_14 = x_72; +x_15 = x_60; x_16 = lean_box(0); goto block_51; } else { -x_8 = x_72; +x_8 = x_74; x_9 = x_53; -x_10 = x_74; -x_11 = x_54; -x_12 = x_57; -x_13 = x_55; -x_14 = x_58; -x_15 = x_71; +x_10 = x_57; +x_11 = x_56; +x_12 = x_58; +x_13 = x_71; +x_14 = x_72; +x_15 = x_60; x_16 = lean_box(0); goto block_51; } @@ -20672,13 +20672,13 @@ else uint8_t x_76; lean_dec(x_63); lean_dec(x_61); -lean_dec(x_60); +lean_dec_ref(x_60); lean_dec(x_59); lean_dec(x_58); lean_dec_ref(x_57); -lean_dec(x_56); -lean_dec_ref(x_55); -lean_dec_ref(x_54); +lean_dec_ref(x_56); +lean_dec(x_55); +lean_dec(x_54); lean_dec_ref(x_53); lean_dec(x_4); lean_dec(x_3); @@ -20704,13 +20704,13 @@ else { uint8_t x_79; lean_dec(x_61); -lean_dec(x_60); +lean_dec_ref(x_60); lean_dec(x_59); lean_dec(x_58); lean_dec_ref(x_57); -lean_dec(x_56); -lean_dec_ref(x_55); -lean_dec_ref(x_54); +lean_dec_ref(x_56); +lean_dec(x_55); +lean_dec(x_54); lean_dec_ref(x_53); lean_dec(x_4); lean_dec(x_3); @@ -20760,14 +20760,14 @@ if (lean_obj_tag(x_86) == 0) lean_object* x_99; x_99 = lean_box(0); x_52 = lean_box(0); -x_53 = x_95; -x_54 = x_96; -x_55 = x_97; -x_56 = x_92; -x_57 = x_87; +x_53 = x_87; +x_54 = x_92; +x_55 = x_94; +x_56 = x_95; +x_57 = x_97; x_58 = x_88; x_59 = x_98; -x_60 = x_94; +x_60 = x_96; x_61 = x_99; goto block_82; } @@ -20778,14 +20778,14 @@ x_100 = !lean_is_exclusive(x_86); if (x_100 == 0) { x_52 = lean_box(0); -x_53 = x_95; -x_54 = x_96; -x_55 = x_97; -x_56 = x_92; -x_57 = x_87; +x_53 = x_87; +x_54 = x_92; +x_55 = x_94; +x_56 = x_95; +x_57 = x_97; x_58 = x_88; x_59 = x_98; -x_60 = x_94; +x_60 = x_96; x_61 = x_86; goto block_82; } @@ -20798,14 +20798,14 @@ lean_dec(x_86); x_102 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_102, 0, x_101); x_52 = lean_box(0); -x_53 = x_95; -x_54 = x_96; -x_55 = x_97; -x_56 = x_92; -x_57 = x_87; +x_53 = x_87; +x_54 = x_92; +x_55 = x_94; +x_56 = x_95; +x_57 = x_97; x_58 = x_88; x_59 = x_98; -x_60 = x_94; +x_60 = x_96; x_61 = x_102; goto block_82; } @@ -20915,19 +20915,19 @@ lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; x_259 = lean_ctor_get(x_258, 0); lean_inc(x_259); lean_dec_ref(x_258); -lean_inc_ref(x_248); -lean_inc(x_241); -lean_inc(x_238); +lean_inc_ref(x_237); +lean_inc(x_243); +lean_inc(x_250); x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_238); -lean_ctor_set(x_260, 1, x_241); -lean_ctor_set(x_260, 2, x_248); +lean_ctor_set(x_260, 0, x_250); +lean_ctor_set(x_260, 1, x_243); +lean_ctor_set(x_260, 2, x_237); lean_inc_ref(x_260); -lean_inc(x_238); -x_261 = l_Lean_Syntax_node1(x_238, x_243, x_260); -lean_inc(x_238); -x_262 = l_Lean_Syntax_node2(x_238, x_246, x_244, x_260); -x_263 = l_Lean_Syntax_node2(x_238, x_247, x_261, x_262); +lean_inc(x_250); +x_261 = l_Lean_Syntax_node1(x_250, x_238, x_260); +lean_inc(x_250); +x_262 = l_Lean_Syntax_node2(x_250, x_245, x_244, x_260); +x_263 = l_Lean_Syntax_node2(x_250, x_246, x_261, x_262); x_264 = lean_unsigned_to_nat(2u); x_265 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_266 = lean_array_push(x_265, x_239); @@ -20945,20 +20945,20 @@ x_272 = lean_ctor_get(x_271, 0); lean_inc(x_272); lean_dec_ref(x_271); x_132 = x_236; -x_133 = x_259; +x_133 = x_269; x_134 = x_237; -x_135 = x_269; -x_136 = x_240; -x_137 = x_264; -x_138 = x_241; -x_139 = x_242; -x_140 = x_257; -x_141 = x_253; -x_142 = x_245; -x_143 = x_248; -x_144 = x_249; -x_145 = x_270; -x_146 = x_250; +x_135 = x_240; +x_136 = x_241; +x_137 = x_242; +x_138 = x_243; +x_139 = x_264; +x_140 = x_247; +x_141 = x_270; +x_142 = x_257; +x_143 = x_259; +x_144 = x_248; +x_145 = x_253; +x_146 = x_249; x_147 = x_272; x_148 = lean_box(0); goto block_229; @@ -20971,20 +20971,20 @@ x_273 = lean_ctor_get(x_234, 0); lean_inc(x_273); lean_dec_ref(x_234); x_132 = x_236; -x_133 = x_259; +x_133 = x_269; x_134 = x_237; -x_135 = x_269; -x_136 = x_240; -x_137 = x_264; -x_138 = x_241; -x_139 = x_242; -x_140 = x_257; -x_141 = x_253; -x_142 = x_245; -x_143 = x_248; -x_144 = x_249; -x_145 = x_270; -x_146 = x_250; +x_135 = x_240; +x_136 = x_241; +x_137 = x_242; +x_138 = x_243; +x_139 = x_264; +x_140 = x_247; +x_141 = x_270; +x_142 = x_257; +x_143 = x_259; +x_144 = x_248; +x_145 = x_253; +x_146 = x_249; x_147 = x_273; x_148 = lean_box(0); goto block_229; @@ -21001,16 +21001,16 @@ lean_dec(x_249); lean_dec_ref(x_248); lean_dec(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec_ref(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec(x_6); @@ -21043,16 +21043,16 @@ lean_dec(x_249); lean_dec_ref(x_248); lean_dec(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec_ref(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -21085,16 +21085,16 @@ lean_dec(x_249); lean_dec_ref(x_248); lean_dec(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec_ref(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -21125,16 +21125,16 @@ lean_dec(x_249); lean_dec_ref(x_248); lean_dec(x_247); lean_dec(x_246); -lean_dec_ref(x_245); +lean_dec(x_245); lean_dec(x_244); lean_dec(x_243); -lean_dec_ref(x_242); -lean_dec(x_241); +lean_dec(x_242); +lean_dec_ref(x_241); lean_dec(x_240); lean_dec(x_239); lean_dec(x_238); lean_dec_ref(x_237); -lean_dec(x_236); +lean_dec_ref(x_236); lean_dec(x_234); lean_dec(x_10); lean_dec_ref(x_9); @@ -21166,68 +21166,68 @@ x_299 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__14; x_300 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__15; x_301 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_302 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; -lean_inc(x_286); +lean_inc(x_290); x_303 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_303, 0, x_286); +lean_ctor_set(x_303, 0, x_290); lean_ctor_set(x_303, 1, x_301); lean_ctor_set(x_303, 2, x_302); lean_inc_ref(x_303); -lean_inc(x_286); -x_304 = l_Lean_Syntax_node1(x_286, x_300, x_303); +lean_inc(x_290); +x_304 = l_Lean_Syntax_node1(x_290, x_300, x_303); x_305 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__16; x_306 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_307 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; -x_308 = l_Lean_addMacroScope(x_291, x_307, x_285); +x_308 = l_Lean_addMacroScope(x_291, x_307, x_286); lean_inc(x_288); -lean_inc(x_286); +lean_inc(x_290); x_309 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_309, 0, x_286); +lean_ctor_set(x_309, 0, x_290); lean_ctor_set(x_309, 1, x_306); lean_ctor_set(x_309, 2, x_308); lean_ctor_set(x_309, 3, x_288); -lean_inc(x_286); -x_310 = l_Lean_Syntax_node2(x_286, x_305, x_309, x_303); -x_311 = l_Lean_Syntax_node2(x_286, x_299, x_304, x_310); +lean_inc(x_290); +x_310 = l_Lean_Syntax_node2(x_290, x_305, x_309, x_303); +x_311 = l_Lean_Syntax_node2(x_290, x_299, x_304, x_310); if (lean_obj_tag(x_234) == 0) { lean_object* x_312; x_312 = l_Lean_getMainModule___at___00__private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabLeanLibCommand_spec__1_spec__4___redArg(x_10); lean_dec_ref(x_312); -x_236 = x_284; -x_237 = x_297; -x_238 = x_294; +x_236 = x_296; +x_237 = x_302; +x_238 = x_300; x_239 = x_311; x_240 = x_288; -x_241 = x_301; -x_242 = x_296; -x_243 = x_300; -x_244 = x_287; -x_245 = x_298; -x_246 = x_305; -x_247 = x_299; -x_248 = x_302; +x_241 = x_298; +x_242 = x_284; +x_243 = x_301; +x_244 = x_285; +x_245 = x_305; +x_246 = x_299; +x_247 = x_287; +x_248 = x_297; x_249 = x_289; -x_250 = x_290; +x_250 = x_294; x_251 = lean_box(0); goto block_283; } else { -x_236 = x_284; -x_237 = x_297; -x_238 = x_294; +x_236 = x_296; +x_237 = x_302; +x_238 = x_300; x_239 = x_311; x_240 = x_288; -x_241 = x_301; -x_242 = x_296; -x_243 = x_300; -x_244 = x_287; -x_245 = x_298; -x_246 = x_305; -x_247 = x_299; -x_248 = x_302; +x_241 = x_298; +x_242 = x_284; +x_243 = x_301; +x_244 = x_285; +x_245 = x_305; +x_246 = x_299; +x_247 = x_287; +x_248 = x_297; x_249 = x_289; -x_250 = x_290; +x_250 = x_294; x_251 = lean_box(0); goto block_283; } @@ -21368,12 +21368,12 @@ x_343 = lean_ctor_get(x_342, 0); lean_inc(x_343); lean_dec_ref(x_342); x_284 = x_331; -x_285 = x_341; -x_286 = x_339; -x_287 = x_337; +x_285 = x_337; +x_286 = x_341; +x_287 = x_329; x_288 = x_328; -x_289 = x_329; -x_290 = x_324; +x_289 = x_324; +x_290 = x_339; x_291 = x_343; x_292 = lean_box(0); goto block_319; @@ -21387,12 +21387,12 @@ lean_dec_ref(x_340); x_345 = lean_ctor_get(x_234, 0); lean_inc(x_345); x_284 = x_331; -x_285 = x_344; -x_286 = x_339; -x_287 = x_337; +x_285 = x_337; +x_286 = x_344; +x_287 = x_329; x_288 = x_328; -x_289 = x_329; -x_290 = x_324; +x_289 = x_324; +x_290 = x_339; x_291 = x_345; x_292 = lean_box(0); goto block_319; @@ -21589,43 +21589,43 @@ return x_364; block_131: { 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_inc_ref(x_23); -x_43 = l_Array_append___redArg(x_23, x_42); +lean_inc_ref(x_16); +x_43 = l_Array_append___redArg(x_16, x_42); lean_dec_ref(x_42); -lean_inc(x_15); -lean_inc(x_36); +lean_inc(x_20); +lean_inc(x_25); x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_36); -lean_ctor_set(x_44, 1, x_15); +lean_ctor_set(x_44, 0, x_25); +lean_ctor_set(x_44, 1, x_20); lean_ctor_set(x_44, 2, x_43); -lean_inc_n(x_21, 6); -lean_inc(x_34); -lean_inc(x_36); -x_45 = l_Lean_Syntax_node7(x_36, x_34, x_44, x_21, x_21, x_21, x_21, x_21, x_21); +lean_inc_n(x_37, 6); +lean_inc(x_22); +lean_inc(x_25); +x_45 = l_Lean_Syntax_node7(x_25, x_22, x_44, x_37, x_37, x_37, x_37, x_37, x_37); x_46 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__9; -lean_inc_ref(x_35); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_47 = l_Lean_Name_mkStr4(x_33, x_28, x_35, x_46); -lean_inc(x_36); +lean_inc_ref(x_18); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_47 = l_Lean_Name_mkStr4(x_15, x_24, x_18, x_46); +lean_inc(x_25); x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_36); +lean_ctor_set(x_48, 0, x_25); lean_ctor_set(x_48, 1, x_46); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_35); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_50 = l_Lean_Name_mkStr4(x_33, x_28, x_35, x_49); +lean_inc_ref(x_18); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_50 = l_Lean_Name_mkStr4(x_15, x_24, x_18, x_49); x_51 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_52 = lean_box(2); -lean_inc(x_15); +lean_inc(x_20); x_53 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_15); +lean_ctor_set(x_53, 1, x_20); lean_ctor_set(x_53, 2, x_51); -x_54 = lean_mk_empty_array_with_capacity(x_14); -lean_inc(x_26); -x_55 = lean_array_push(x_54, x_26); +x_54 = lean_mk_empty_array_with_capacity(x_34); +lean_inc(x_27); +x_55 = lean_array_push(x_54, x_27); x_56 = lean_array_push(x_55, x_53); lean_inc(x_50); x_57 = lean_alloc_ctor(1, 3, 0); @@ -21633,194 +21633,194 @@ lean_ctor_set(x_57, 0, x_52); lean_ctor_set(x_57, 1, x_50); lean_ctor_set(x_57, 2, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_35); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_59 = l_Lean_Name_mkStr4(x_33, x_28, x_35, x_58); +lean_inc_ref(x_18); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_59 = l_Lean_Name_mkStr4(x_15, x_24, x_18, x_58); x_60 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_22); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_61 = l_Lean_Name_mkStr4(x_33, x_28, x_22, x_60); -lean_inc(x_39); +lean_inc_ref(x_31); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_61 = l_Lean_Name_mkStr4(x_15, x_24, x_31, x_60); +lean_inc(x_29); lean_inc(x_61); -lean_inc(x_36); -x_62 = l_Lean_Syntax_node2(x_36, x_61, x_39, x_38); -lean_inc(x_15); -lean_inc(x_36); -x_63 = l_Lean_Syntax_node1(x_36, x_15, x_62); -lean_inc(x_21); +lean_inc(x_25); +x_62 = l_Lean_Syntax_node2(x_25, x_61, x_29, x_40); +lean_inc(x_20); +lean_inc(x_25); +x_63 = l_Lean_Syntax_node1(x_25, x_20, x_62); +lean_inc(x_37); lean_inc(x_59); -lean_inc(x_36); -x_64 = l_Lean_Syntax_node2(x_36, x_59, x_21, x_63); +lean_inc(x_25); +x_64 = l_Lean_Syntax_node2(x_25, x_59, x_37, x_63); x_65 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__60; -lean_inc_ref(x_35); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_66 = l_Lean_Name_mkStr4(x_33, x_28, x_35, x_65); +lean_inc_ref(x_18); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_66 = l_Lean_Name_mkStr4(x_15, x_24, x_18, x_65); x_67 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__1; x_68 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__2; -lean_inc_ref(x_31); -x_69 = l_Lean_Name_mkStr3(x_31, x_40, x_68); -lean_inc(x_29); +lean_inc_ref(x_39); +x_69 = l_Lean_Name_mkStr3(x_39, x_12, x_68); +lean_inc(x_26); lean_inc(x_69); -lean_inc(x_30); -x_70 = l_Lean_addMacroScope(x_30, x_69, x_29); -lean_inc(x_37); +lean_inc(x_13); +x_70 = l_Lean_addMacroScope(x_13, x_69, x_26); +lean_inc(x_32); x_71 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_37); -lean_inc(x_32); +lean_ctor_set(x_71, 1, x_32); +lean_inc(x_17); x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_32); -lean_inc(x_36); +lean_ctor_set(x_72, 1, x_17); +lean_inc(x_25); x_73 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_73, 0, x_36); +lean_ctor_set(x_73, 0, x_25); lean_ctor_set(x_73, 1, x_67); lean_ctor_set(x_73, 2, x_70); lean_ctor_set(x_73, 3, x_72); -lean_inc(x_15); -lean_inc(x_36); -x_74 = l_Lean_Syntax_node4(x_36, x_15, x_13, x_27, x_41, x_24); -lean_inc(x_36); -x_75 = l_Lean_Syntax_node2(x_36, x_16, x_73, x_74); +lean_inc(x_20); +lean_inc(x_25); +x_74 = l_Lean_Syntax_node4(x_25, x_20, x_36, x_33, x_23, x_38); +lean_inc(x_25); +x_75 = l_Lean_Syntax_node2(x_25, x_21, x_73, x_74); x_76 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__62; x_77 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__63; -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_78 = l_Lean_Name_mkStr4(x_33, x_28, x_76, x_77); -lean_inc_n(x_21, 2); -lean_inc(x_36); -x_79 = l_Lean_Syntax_node2(x_36, x_78, x_21, x_21); -lean_inc(x_21); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_78 = l_Lean_Name_mkStr4(x_15, x_24, x_76, x_77); +lean_inc_n(x_37, 2); +lean_inc(x_25); +x_79 = l_Lean_Syntax_node2(x_25, x_78, x_37, x_37); +lean_inc(x_37); lean_inc(x_79); -lean_inc(x_18); +lean_inc(x_35); lean_inc(x_66); -lean_inc(x_36); -x_80 = l_Lean_Syntax_node4(x_36, x_66, x_18, x_75, x_79, x_21); -lean_inc(x_36); -x_81 = l_Lean_Syntax_node4(x_36, x_47, x_48, x_57, x_64, x_80); +lean_inc(x_25); +x_80 = l_Lean_Syntax_node4(x_25, x_66, x_35, x_75, x_79, x_37); +lean_inc(x_25); +x_81 = l_Lean_Syntax_node4(x_25, x_47, x_48, x_57, x_64, x_80); lean_inc(x_19); -lean_inc(x_36); -x_82 = l_Lean_Syntax_node2(x_36, x_19, x_45, x_81); +lean_inc(x_25); +x_82 = l_Lean_Syntax_node2(x_25, x_19, x_45, x_81); x_83 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_22); -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_84 = l_Lean_Name_mkStr4(x_33, x_28, x_22, x_83); +lean_inc_ref(x_31); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_84 = l_Lean_Name_mkStr4(x_15, x_24, x_31, x_83); x_85 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_36); +lean_inc(x_25); x_86 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_86, 0, x_36); +lean_ctor_set(x_86, 0, x_25); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Syntax_SepArray_ofElems(x_20, x_12); -lean_dec_ref(x_12); -x_88 = l_Array_append___redArg(x_23, x_87); +x_87 = l_Lean_Syntax_SepArray_ofElems(x_30, x_14); +lean_dec_ref(x_14); +x_88 = l_Array_append___redArg(x_16, x_87); lean_dec_ref(x_87); -lean_inc(x_15); -lean_inc(x_36); +lean_inc(x_20); +lean_inc(x_25); x_89 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_89, 0, x_36); -lean_ctor_set(x_89, 1, x_15); +lean_ctor_set(x_89, 0, x_25); +lean_ctor_set(x_89, 1, x_20); lean_ctor_set(x_89, 2, x_88); x_90 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_36); +lean_inc(x_25); x_91 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_91, 0, x_36); +lean_ctor_set(x_91, 0, x_25); lean_ctor_set(x_91, 1, x_90); -lean_inc(x_36); -x_92 = l_Lean_Syntax_node3(x_36, x_84, x_86, x_89, x_91); -lean_inc(x_15); -lean_inc(x_36); -x_93 = l_Lean_Syntax_node1(x_36, x_15, x_92); -lean_inc_n(x_21, 6); -lean_inc(x_36); -x_94 = l_Lean_Syntax_node7(x_36, x_34, x_21, x_93, x_21, x_21, x_21, x_21, x_21); +lean_inc(x_25); +x_92 = l_Lean_Syntax_node3(x_25, x_84, x_86, x_89, x_91); +lean_inc(x_20); +lean_inc(x_25); +x_93 = l_Lean_Syntax_node1(x_25, x_20, x_92); +lean_inc_n(x_37, 6); +lean_inc(x_25); +x_94 = l_Lean_Syntax_node7(x_25, x_22, x_37, x_93, x_37, x_37, x_37, x_37, x_37); x_95 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_28); -lean_inc_ref(x_33); -x_96 = l_Lean_Name_mkStr4(x_33, x_28, x_35, x_95); +lean_inc_ref(x_24); +lean_inc_ref(x_15); +x_96 = l_Lean_Name_mkStr4(x_15, x_24, x_18, x_95); x_97 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_36); +lean_inc(x_25); x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_36); +lean_ctor_set(x_98, 0, x_25); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_100 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_29); -lean_inc(x_30); -x_101 = l_Lean_addMacroScope(x_30, x_100, x_29); -lean_inc(x_32); -lean_inc(x_36); +lean_inc(x_26); +lean_inc(x_13); +x_101 = l_Lean_addMacroScope(x_13, x_100, x_26); +lean_inc(x_17); +lean_inc(x_25); x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_36); +lean_ctor_set(x_102, 0, x_25); lean_ctor_set(x_102, 1, x_99); lean_ctor_set(x_102, 2, x_101); -lean_ctor_set(x_102, 3, x_32); -lean_inc(x_21); -lean_inc(x_36); -x_103 = l_Lean_Syntax_node2(x_36, x_50, x_102, x_21); +lean_ctor_set(x_102, 3, x_17); +lean_inc(x_37); +lean_inc(x_25); +x_103 = l_Lean_Syntax_node2(x_25, x_50, x_102, x_37); x_104 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__5; x_105 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_106 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_29); -lean_inc(x_30); -x_107 = l_Lean_addMacroScope(x_30, x_106, x_29); -x_108 = l_Lean_Name_mkStr2(x_31, x_104); +lean_inc(x_26); +lean_inc(x_13); +x_107 = l_Lean_addMacroScope(x_13, x_106, x_26); +x_108 = l_Lean_Name_mkStr2(x_39, x_104); lean_inc(x_108); x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_37); +lean_ctor_set(x_109, 1, x_32); x_110 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_110, 0, x_108); -lean_inc(x_32); +lean_inc(x_17); x_111 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_32); +lean_ctor_set(x_111, 1, x_17); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_109); lean_ctor_set(x_112, 1, x_111); -lean_inc(x_36); +lean_inc(x_25); x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_36); +lean_ctor_set(x_113, 0, x_25); lean_ctor_set(x_113, 1, x_105); lean_ctor_set(x_113, 2, x_107); lean_ctor_set(x_113, 3, x_112); -lean_inc(x_36); -x_114 = l_Lean_Syntax_node2(x_36, x_61, x_39, x_113); -lean_inc(x_15); -lean_inc(x_36); -x_115 = l_Lean_Syntax_node1(x_36, x_15, x_114); -lean_inc(x_21); -lean_inc(x_36); -x_116 = l_Lean_Syntax_node2(x_36, x_59, x_21, x_115); +lean_inc(x_25); +x_114 = l_Lean_Syntax_node2(x_25, x_61, x_29, x_113); +lean_inc(x_20); +lean_inc(x_25); +x_115 = l_Lean_Syntax_node1(x_25, x_20, x_114); +lean_inc(x_37); +lean_inc(x_25); +x_116 = l_Lean_Syntax_node2(x_25, x_59, x_37, x_115); x_117 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_118 = l_Lean_Name_mkStr4(x_33, x_28, x_22, x_117); +x_118 = l_Lean_Name_mkStr4(x_15, x_24, x_31, x_117); x_119 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_36); +lean_inc(x_25); x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_36); +lean_ctor_set(x_120, 0, x_25); lean_ctor_set(x_120, 1, x_119); x_121 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_122 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_123 = l_Lean_addMacroScope(x_30, x_122, x_29); -lean_inc(x_36); +x_123 = l_Lean_addMacroScope(x_13, x_122, x_26); +lean_inc(x_25); x_124 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_124, 0, x_36); +lean_ctor_set(x_124, 0, x_25); lean_ctor_set(x_124, 1, x_121); lean_ctor_set(x_124, 2, x_123); -lean_ctor_set(x_124, 3, x_32); -lean_inc(x_36); -x_125 = l_Lean_Syntax_node3(x_36, x_118, x_26, x_120, x_124); -lean_inc(x_21); -lean_inc(x_36); -x_126 = l_Lean_Syntax_node4(x_36, x_66, x_18, x_125, x_79, x_21); -lean_inc(x_36); -x_127 = l_Lean_Syntax_node5(x_36, x_96, x_98, x_103, x_116, x_126, x_21); -lean_inc(x_36); -x_128 = l_Lean_Syntax_node2(x_36, x_19, x_94, x_127); -x_129 = l_Lean_Syntax_node3(x_36, x_15, x_17, x_82, x_128); +lean_ctor_set(x_124, 3, x_17); +lean_inc(x_25); +x_125 = l_Lean_Syntax_node3(x_25, x_118, x_27, x_120, x_124); +lean_inc(x_37); +lean_inc(x_25); +x_126 = l_Lean_Syntax_node4(x_25, x_66, x_35, x_125, x_79, x_37); +lean_inc(x_25); +x_127 = l_Lean_Syntax_node5(x_25, x_96, x_98, x_103, x_116, x_126, x_37); +lean_inc(x_25); +x_128 = l_Lean_Syntax_node2(x_25, x_19, x_94, x_127); +x_129 = l_Lean_Syntax_node3(x_25, x_20, x_28, x_82, x_128); x_130 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_130, 0, x_129); return x_130; @@ -21830,91 +21830,91 @@ return x_130; 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; x_149 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__0; x_150 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; -lean_inc_ref(x_143); +lean_inc_ref(x_134); lean_inc(x_138); -lean_inc(x_140); +lean_inc(x_142); x_151 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_151, 0, x_140); +lean_ctor_set(x_151, 0, x_142); lean_ctor_set(x_151, 1, x_138); -lean_ctor_set(x_151, 2, x_143); +lean_ctor_set(x_151, 2, x_134); x_152 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; -lean_inc(x_140); +lean_inc(x_142); x_153 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_153, 0, x_140); +lean_ctor_set(x_153, 0, x_142); lean_ctor_set(x_153, 1, x_152); x_154 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_140); +lean_inc(x_142); x_155 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_155, 0, x_140); +lean_ctor_set(x_155, 0, x_142); lean_ctor_set(x_155, 1, x_154); x_156 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__30; x_157 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__31; -lean_inc(x_133); +lean_inc(x_143); lean_inc(x_147); -x_158 = l_Lean_addMacroScope(x_147, x_157, x_133); +x_158 = l_Lean_addMacroScope(x_147, x_157, x_143); x_159 = lean_box(0); x_160 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__3; -lean_inc(x_136); +lean_inc(x_135); x_161 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_136); -lean_inc(x_140); +lean_ctor_set(x_161, 1, x_135); +lean_inc(x_142); x_162 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_162, 0, x_140); +lean_ctor_set(x_162, 0, x_142); lean_ctor_set(x_162, 1, x_156); lean_ctor_set(x_162, 2, x_158); lean_ctor_set(x_162, 3, x_161); x_163 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_142); -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_164 = l_Lean_Name_mkStr4(x_139, x_134, x_142, x_163); +lean_inc_ref(x_136); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_164 = l_Lean_Name_mkStr4(x_132, x_144, x_136, x_163); x_165 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_142); -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_166 = l_Lean_Name_mkStr4(x_139, x_134, x_142, x_165); +lean_inc_ref(x_136); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_166 = l_Lean_Name_mkStr4(x_132, x_144, x_136, x_165); x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; -lean_inc(x_140); +lean_inc(x_142); x_168 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_168, 0, x_140); +lean_ctor_set(x_168, 0, x_142); lean_ctor_set(x_168, 1, x_167); x_169 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__25; x_170 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__27; x_171 = lean_box(0); -lean_inc(x_133); +lean_inc(x_143); lean_inc(x_147); -x_172 = l_Lean_addMacroScope(x_147, x_171, x_133); +x_172 = l_Lean_addMacroScope(x_147, x_171, x_143); x_173 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__1; x_174 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__59; -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_176 = l_Lean_Name_mkStr3(x_139, x_134, x_175); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_176 = l_Lean_Name_mkStr3(x_132, x_144, x_175); x_177 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_177, 0, x_176); x_178 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_139); -x_179 = l_Lean_Name_mkStr3(x_139, x_178, x_175); +lean_inc_ref(x_132); +x_179 = l_Lean_Name_mkStr3(x_132, x_178, x_175); x_180 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_180, 0, x_179); -lean_inc_ref(x_139); -x_181 = l_Lean_Name_mkStr2(x_139, x_178); +lean_inc_ref(x_132); +x_181 = l_Lean_Name_mkStr2(x_132, x_178); x_182 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_182, 0, x_181); -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_183 = l_Lean_Name_mkStr2(x_139, x_134); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_183 = l_Lean_Name_mkStr2(x_132, x_144); x_184 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_184, 0, x_183); -lean_inc_ref(x_139); -x_185 = l_Lean_Name_mkStr1(x_139); +lean_inc_ref(x_132); +x_185 = l_Lean_Name_mkStr1(x_132); x_186 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_186, 0, x_185); -lean_inc(x_136); +lean_inc(x_135); x_187 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_187, 0, x_186); -lean_ctor_set(x_187, 1, x_136); +lean_ctor_set(x_187, 1, x_135); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_184); lean_ctor_set(x_188, 1, x_187); @@ -21930,95 +21930,95 @@ lean_ctor_set(x_191, 1, x_190); x_192 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_192, 0, x_174); lean_ctor_set(x_192, 1, x_191); -lean_inc(x_140); +lean_inc(x_142); x_193 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_193, 0, x_140); +lean_ctor_set(x_193, 0, x_142); lean_ctor_set(x_193, 1, x_170); lean_ctor_set(x_193, 2, x_172); lean_ctor_set(x_193, 3, x_192); -lean_inc(x_140); -x_194 = l_Lean_Syntax_node1(x_140, x_169, x_193); -lean_inc(x_140); -x_195 = l_Lean_Syntax_node2(x_140, x_166, x_168, x_194); +lean_inc(x_142); +x_194 = l_Lean_Syntax_node1(x_142, x_169, x_193); +lean_inc(x_142); +x_195 = l_Lean_Syntax_node2(x_142, x_166, x_168, x_194); x_196 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__37; x_197 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__38; -lean_inc(x_140); +lean_inc(x_142); x_198 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_198, 0, x_140); +lean_ctor_set(x_198, 0, x_142); lean_ctor_set(x_198, 1, x_197); -lean_inc(x_140); -x_199 = l_Lean_Syntax_node1(x_140, x_196, x_198); +lean_inc(x_142); +x_199 = l_Lean_Syntax_node1(x_142, x_196, x_198); x_200 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__7; -lean_inc(x_140); +lean_inc(x_142); x_201 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_201, 0, x_140); +lean_ctor_set(x_201, 0, x_142); lean_ctor_set(x_201, 1, x_200); -lean_inc(x_132); +lean_inc(x_137); lean_inc(x_138); -lean_inc(x_140); -x_202 = l_Lean_Syntax_node1(x_140, x_138, x_132); +lean_inc(x_142); +x_202 = l_Lean_Syntax_node1(x_142, x_138, x_137); lean_inc(x_199); lean_inc(x_138); -lean_inc(x_140); -x_203 = l_Lean_Syntax_node3(x_140, x_138, x_199, x_201, x_202); +lean_inc(x_142); +x_203 = l_Lean_Syntax_node3(x_142, x_138, x_199, x_201, x_202); x_204 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; -lean_inc(x_140); +lean_inc(x_142); x_205 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_205, 0, x_140); +lean_ctor_set(x_205, 0, x_142); lean_ctor_set(x_205, 1, x_204); -lean_inc(x_140); -x_206 = l_Lean_Syntax_node3(x_140, x_164, x_195, x_203, x_205); +lean_inc(x_142); +x_206 = l_Lean_Syntax_node3(x_142, x_164, x_195, x_203, x_205); x_207 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__14; -lean_inc(x_140); +lean_inc(x_142); x_208 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_208, 0, x_140); +lean_ctor_set(x_208, 0, x_142); lean_ctor_set(x_208, 1, x_207); x_209 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_142); -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_210 = l_Lean_Name_mkStr4(x_139, x_134, x_142, x_209); +lean_inc_ref(x_136); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_210 = l_Lean_Name_mkStr4(x_132, x_144, x_136, x_209); x_211 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_212 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; -lean_inc(x_133); +lean_inc(x_143); lean_inc(x_147); -x_213 = l_Lean_addMacroScope(x_147, x_212, x_133); +x_213 = l_Lean_addMacroScope(x_147, x_212, x_143); x_214 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__8; x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_136); +lean_inc(x_135); x_216 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_136); +lean_ctor_set(x_216, 1, x_135); x_217 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_217, 0, x_214); lean_ctor_set(x_217, 1, x_216); -lean_inc(x_140); +lean_inc(x_142); x_218 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_218, 0, x_140); +lean_ctor_set(x_218, 0, x_142); lean_ctor_set(x_218, 1, x_211); lean_ctor_set(x_218, 2, x_213); lean_ctor_set(x_218, 3, x_217); -lean_inc(x_145); +lean_inc(x_141); lean_inc(x_138); -lean_inc(x_140); -x_219 = l_Lean_Syntax_node1(x_140, x_138, x_145); +lean_inc(x_142); +x_219 = l_Lean_Syntax_node1(x_142, x_138, x_141); lean_inc(x_210); -lean_inc(x_140); -x_220 = l_Lean_Syntax_node2(x_140, x_210, x_218, x_219); +lean_inc(x_142); +x_220 = l_Lean_Syntax_node2(x_142, x_210, x_218, x_219); lean_inc_ref(x_208); lean_inc_ref(x_155); lean_inc(x_146); lean_inc_ref(x_151); -lean_inc(x_140); -x_221 = l_Lean_Syntax_node8(x_140, x_150, x_151, x_153, x_146, x_155, x_162, x_206, x_208, x_220); +lean_inc(x_142); +x_221 = l_Lean_Syntax_node8(x_142, x_150, x_151, x_153, x_146, x_155, x_162, x_206, x_208, x_220); x_222 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_223 = l_Lean_Name_mkStr4(x_139, x_134, x_175, x_222); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_223 = l_Lean_Name_mkStr4(x_132, x_144, x_175, x_222); x_224 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_134); -lean_inc_ref(x_139); -x_225 = l_Lean_Name_mkStr4(x_139, x_134, x_175, x_224); +lean_inc_ref(x_144); +lean_inc_ref(x_132); +x_225 = l_Lean_Name_mkStr4(x_132, x_144, x_175, x_224); if (lean_obj_tag(x_5) == 1) { lean_object* x_226; lean_object* x_227; @@ -22026,36 +22026,36 @@ x_226 = lean_ctor_get(x_5, 0); lean_inc(x_226); lean_dec_ref(x_5); x_227 = l_Array_mkArray1___redArg(x_226); -x_12 = x_135; -x_13 = x_199; -x_14 = x_137; -x_15 = x_138; -x_16 = x_210; -x_17 = x_221; -x_18 = x_208; +x_12 = x_173; +x_13 = x_147; +x_14 = x_133; +x_15 = x_132; +x_16 = x_134; +x_17 = x_135; +x_18 = x_175; x_19 = x_223; -x_20 = x_200; -x_21 = x_151; -x_22 = x_142; -x_23 = x_143; +x_20 = x_138; +x_21 = x_210; +x_22 = x_225; +x_23 = x_141; x_24 = x_144; -x_25 = lean_box(0); -x_26 = x_146; -x_27 = x_132; -x_28 = x_134; -x_29 = x_133; -x_30 = x_147; -x_31 = x_149; -x_32 = x_136; -x_33 = x_139; -x_34 = x_225; -x_35 = x_175; -x_36 = x_140; -x_37 = x_159; -x_38 = x_141; -x_39 = x_155; -x_40 = x_173; -x_41 = x_145; +x_25 = x_142; +x_26 = x_143; +x_27 = x_146; +x_28 = x_221; +x_29 = x_155; +x_30 = x_200; +x_31 = x_136; +x_32 = x_159; +x_33 = x_137; +x_34 = x_139; +x_35 = x_208; +x_36 = x_199; +x_37 = x_151; +x_38 = x_140; +x_39 = x_149; +x_40 = x_145; +x_41 = lean_box(0); x_42 = x_227; goto block_131; } @@ -22064,36 +22064,36 @@ else lean_object* x_228; lean_dec(x_5); x_228 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_12 = x_135; -x_13 = x_199; -x_14 = x_137; -x_15 = x_138; -x_16 = x_210; -x_17 = x_221; -x_18 = x_208; +x_12 = x_173; +x_13 = x_147; +x_14 = x_133; +x_15 = x_132; +x_16 = x_134; +x_17 = x_135; +x_18 = x_175; x_19 = x_223; -x_20 = x_200; -x_21 = x_151; -x_22 = x_142; -x_23 = x_143; +x_20 = x_138; +x_21 = x_210; +x_22 = x_225; +x_23 = x_141; x_24 = x_144; -x_25 = lean_box(0); -x_26 = x_146; -x_27 = x_132; -x_28 = x_134; -x_29 = x_133; -x_30 = x_147; -x_31 = x_149; -x_32 = x_136; -x_33 = x_139; -x_34 = x_225; -x_35 = x_175; -x_36 = x_140; -x_37 = x_159; -x_38 = x_141; -x_39 = x_155; -x_40 = x_173; -x_41 = x_145; +x_25 = x_142; +x_26 = x_143; +x_27 = x_146; +x_28 = x_221; +x_29 = x_155; +x_30 = x_200; +x_31 = x_136; +x_32 = x_159; +x_33 = x_137; +x_34 = x_139; +x_35 = x_208; +x_36 = x_199; +x_37 = x_151; +x_38 = x_140; +x_39 = x_149; +x_40 = x_145; +x_41 = lean_box(0); x_42 = x_228; goto block_131; } @@ -22184,7 +22184,7 @@ lean_dec(x_14); lean_ctor_set(x_2, 7, x_29); lean_inc(x_3); lean_inc_ref(x_2); -x_30 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputDirCommand_spec__0(x_27, x_28, x_28, x_26, x_21, x_19, x_20, x_18, x_2, x_3); +x_30 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputDirCommand_spec__0(x_27, x_28, x_28, x_26, x_21, x_20, x_19, x_18, x_2, x_3); if (lean_obj_tag(x_30) == 0) { lean_object* x_31; lean_object* x_32; lean_object* x_33; @@ -22263,7 +22263,7 @@ lean_ctor_set(x_51, 9, x_45); lean_ctor_set_uint8(x_51, sizeof(void*)*10, x_46); lean_inc(x_3); lean_inc_ref(x_51); -x_52 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputDirCommand_spec__0(x_48, x_49, x_49, x_47, x_21, x_19, x_20, x_18, x_51, x_3); +x_52 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___at___00__private_Lake_DSL_Targets_0__Lake_DSL_elabInputDirCommand_spec__0(x_48, x_49, x_49, x_47, x_21, x_20, x_19, x_18, x_51, x_3); if (lean_obj_tag(x_52) == 0) { lean_object* x_53; lean_object* x_54; lean_object* x_55; @@ -22338,8 +22338,8 @@ if (lean_obj_tag(x_65) == 0) { lean_object* x_66; x_66 = lean_box(0); -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_66; goto block_62; } @@ -22349,8 +22349,8 @@ uint8_t x_67; x_67 = !lean_is_exclusive(x_65); if (x_67 == 0) { -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_65; goto block_62; } @@ -22362,8 +22362,8 @@ lean_inc(x_68); lean_dec(x_65); x_69 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_69, 0, x_68); -x_19 = x_64; -x_20 = x_63; +x_19 = x_63; +x_20 = x_64; x_21 = x_69; goto block_62; } @@ -22830,44 +22830,44 @@ goto block_522; block_124: { 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_inc_ref(x_24); -x_42 = l_Array_append___redArg(x_24, x_41); +lean_inc_ref(x_36); +x_42 = l_Array_append___redArg(x_36, x_41); lean_dec_ref(x_41); -lean_inc(x_39); -lean_inc(x_23); +lean_inc(x_24); +lean_inc(x_19); x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_23); -lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 0, x_19); +lean_ctor_set(x_43, 1, x_24); lean_ctor_set(x_43, 2, x_42); -lean_inc_n(x_38, 6); -lean_inc(x_31); -lean_inc(x_23); -x_44 = l_Lean_Syntax_node7(x_23, x_31, x_43, x_38, x_38, x_38, x_38, x_38, x_38); +lean_inc_n(x_32, 6); +lean_inc(x_39); +lean_inc(x_19); +x_44 = l_Lean_Syntax_node7(x_19, x_39, x_43, x_32, x_32, x_32, x_32, x_32, x_32); x_45 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__0; -lean_inc_ref(x_19); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_46 = l_Lean_Name_mkStr4(x_28, x_29, x_19, x_45); +lean_inc_ref(x_25); +lean_inc_ref(x_37); +lean_inc_ref(x_16); +x_46 = l_Lean_Name_mkStr4(x_16, x_37, x_25, x_45); x_47 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__1; -lean_inc(x_23); +lean_inc(x_19); x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_23); +lean_ctor_set(x_48, 0, x_19); lean_ctor_set(x_48, 1, x_47); x_49 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__10; -lean_inc_ref(x_19); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_50 = l_Lean_Name_mkStr4(x_28, x_29, x_19, x_49); +lean_inc_ref(x_25); +lean_inc_ref(x_37); +lean_inc_ref(x_16); +x_50 = l_Lean_Name_mkStr4(x_16, x_37, x_25, x_49); x_51 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__11; x_52 = lean_box(2); -lean_inc(x_39); +lean_inc(x_24); x_53 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_39); +lean_ctor_set(x_53, 1, x_24); lean_ctor_set(x_53, 2, x_51); x_54 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; -lean_inc(x_34); -x_55 = lean_array_push(x_54, x_34); +lean_inc(x_17); +x_55 = lean_array_push(x_54, x_17); x_56 = lean_array_push(x_55, x_53); lean_inc(x_50); x_57 = lean_alloc_ctor(1, 3, 0); @@ -22875,287 +22875,287 @@ lean_ctor_set(x_57, 0, x_52); lean_ctor_set(x_57, 1, x_50); lean_ctor_set(x_57, 2, x_56); x_58 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__13; -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_59 = l_Lean_Name_mkStr4(x_28, x_29, x_19, x_58); +lean_inc_ref(x_37); +lean_inc_ref(x_16); +x_59 = l_Lean_Name_mkStr4(x_16, x_37, x_25, x_58); x_60 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__4; x_61 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__5; -lean_inc(x_15); -lean_inc(x_32); -x_62 = l_Lean_addMacroScope(x_32, x_61, x_15); +lean_inc(x_13); +lean_inc(x_35); +x_62 = l_Lean_addMacroScope(x_35, x_61, x_13); x_63 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__6; -lean_inc(x_14); +lean_inc(x_31); x_64 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_14); -lean_inc(x_18); +lean_ctor_set(x_64, 1, x_31); +lean_inc(x_33); x_65 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_18); -lean_inc(x_23); +lean_ctor_set(x_65, 1, x_33); +lean_inc(x_19); x_66 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_66, 0, x_23); +lean_ctor_set(x_66, 0, x_19); lean_ctor_set(x_66, 1, x_60); lean_ctor_set(x_66, 2, x_62); lean_ctor_set(x_66, 3, x_65); -lean_inc(x_35); -lean_inc(x_30); -lean_inc(x_23); -x_67 = l_Lean_Syntax_node2(x_23, x_30, x_35, x_66); -lean_inc(x_39); +lean_inc(x_40); lean_inc(x_23); -x_68 = l_Lean_Syntax_node1(x_23, x_39, x_67); -lean_inc(x_38); +lean_inc(x_19); +x_67 = l_Lean_Syntax_node2(x_19, x_23, x_40, x_66); +lean_inc(x_24); +lean_inc(x_19); +x_68 = l_Lean_Syntax_node1(x_19, x_24, x_67); +lean_inc(x_32); lean_inc(x_59); -lean_inc(x_23); -x_69 = l_Lean_Syntax_node2(x_23, x_59, x_38, x_68); +lean_inc(x_19); +x_69 = l_Lean_Syntax_node2(x_19, x_59, x_32, x_68); x_70 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__8; x_71 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__10; -lean_inc(x_15); -lean_inc(x_32); -x_72 = l_Lean_addMacroScope(x_32, x_71, x_15); -lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_35); +x_72 = l_Lean_addMacroScope(x_35, x_71, x_13); +lean_inc(x_31); x_73 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_14); -lean_inc(x_18); +lean_ctor_set(x_73, 1, x_31); +lean_inc(x_33); x_74 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_18); -lean_inc(x_23); +lean_ctor_set(x_74, 1, x_33); +lean_inc(x_19); x_75 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_75, 0, x_23); +lean_ctor_set(x_75, 0, x_19); lean_ctor_set(x_75, 1, x_70); lean_ctor_set(x_75, 2, x_72); lean_ctor_set(x_75, 3, x_74); -lean_inc(x_39); -lean_inc(x_23); -x_76 = l_Lean_Syntax_node2(x_23, x_39, x_20, x_21); -lean_inc(x_23); -x_77 = l_Lean_Syntax_node2(x_23, x_22, x_75, x_76); -lean_inc(x_38); -lean_inc(x_25); -lean_inc(x_33); -lean_inc(x_26); -lean_inc(x_23); -x_78 = l_Lean_Syntax_node4(x_23, x_26, x_33, x_77, x_25, x_38); -lean_inc(x_38); +lean_inc(x_24); +lean_inc(x_19); +x_76 = l_Lean_Syntax_node2(x_19, x_24, x_14, x_27); +lean_inc(x_19); +x_77 = l_Lean_Syntax_node2(x_19, x_28, x_75, x_76); +lean_inc(x_32); +lean_inc(x_20); +lean_inc(x_18); +lean_inc(x_30); +lean_inc(x_19); +x_78 = l_Lean_Syntax_node4(x_19, x_30, x_18, x_77, x_20, x_32); +lean_inc(x_32); lean_inc_ref(x_48); lean_inc(x_46); -lean_inc(x_23); -x_79 = l_Lean_Syntax_node5(x_23, x_46, x_48, x_57, x_69, x_78, x_38); -lean_inc(x_13); -lean_inc(x_23); -x_80 = l_Lean_Syntax_node2(x_23, x_13, x_44, x_79); +lean_inc(x_19); +x_79 = l_Lean_Syntax_node5(x_19, x_46, x_48, x_57, x_69, x_78, x_32); +lean_inc(x_38); +lean_inc(x_19); +x_80 = l_Lean_Syntax_node2(x_19, x_38, x_44, x_79); x_81 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__5; -lean_inc_ref(x_40); -lean_inc_ref(x_29); -lean_inc_ref(x_28); -x_82 = l_Lean_Name_mkStr4(x_28, x_29, x_40, x_81); +lean_inc_ref(x_15); +lean_inc_ref(x_37); +lean_inc_ref(x_16); +x_82 = l_Lean_Name_mkStr4(x_16, x_37, x_15, x_81); x_83 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__6; -lean_inc(x_23); +lean_inc(x_19); x_84 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_84, 0, x_23); +lean_ctor_set(x_84, 0, x_19); lean_ctor_set(x_84, 1, x_83); -x_85 = l_Lean_Syntax_SepArray_ofElems(x_27, x_36); -lean_dec_ref(x_36); -x_86 = l_Array_append___redArg(x_24, x_85); +x_85 = l_Lean_Syntax_SepArray_ofElems(x_26, x_21); +lean_dec_ref(x_21); +x_86 = l_Array_append___redArg(x_36, x_85); lean_dec_ref(x_85); -lean_inc(x_39); -lean_inc(x_23); +lean_inc(x_24); +lean_inc(x_19); x_87 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_87, 0, x_23); -lean_ctor_set(x_87, 1, x_39); +lean_ctor_set(x_87, 0, x_19); +lean_ctor_set(x_87, 1, x_24); lean_ctor_set(x_87, 2, x_86); x_88 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__8; -lean_inc(x_23); +lean_inc(x_19); x_89 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_89, 0, x_23); +lean_ctor_set(x_89, 0, x_19); lean_ctor_set(x_89, 1, x_88); -lean_inc(x_23); -x_90 = l_Lean_Syntax_node3(x_23, x_82, x_84, x_87, x_89); -lean_inc(x_39); -lean_inc(x_23); -x_91 = l_Lean_Syntax_node1(x_23, x_39, x_90); -lean_inc_n(x_38, 6); -lean_inc(x_23); -x_92 = l_Lean_Syntax_node7(x_23, x_31, x_38, x_91, x_38, x_38, x_38, x_38, x_38); +lean_inc(x_19); +x_90 = l_Lean_Syntax_node3(x_19, x_82, x_84, x_87, x_89); +lean_inc(x_24); +lean_inc(x_19); +x_91 = l_Lean_Syntax_node1(x_19, x_24, x_90); +lean_inc_n(x_32, 6); +lean_inc(x_19); +x_92 = l_Lean_Syntax_node7(x_19, x_39, x_32, x_91, x_32, x_32, x_32, x_32, x_32); x_93 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__3; x_94 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__4; -lean_inc(x_15); -lean_inc(x_32); -x_95 = l_Lean_addMacroScope(x_32, x_94, x_15); -lean_inc(x_18); -lean_inc(x_23); +lean_inc(x_13); +lean_inc(x_35); +x_95 = l_Lean_addMacroScope(x_35, x_94, x_13); +lean_inc(x_33); +lean_inc(x_19); x_96 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_96, 0, x_23); +lean_ctor_set(x_96, 0, x_19); lean_ctor_set(x_96, 1, x_93); lean_ctor_set(x_96, 2, x_95); -lean_ctor_set(x_96, 3, x_18); -lean_inc(x_38); -lean_inc(x_23); -x_97 = l_Lean_Syntax_node2(x_23, x_50, x_96, x_38); +lean_ctor_set(x_96, 3, x_33); +lean_inc(x_32); +lean_inc(x_19); +x_97 = l_Lean_Syntax_node2(x_19, x_50, x_96, x_32); x_98 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__6; x_99 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__7; -lean_inc(x_15); -lean_inc(x_32); -x_100 = l_Lean_addMacroScope(x_32, x_99, x_15); +lean_inc(x_13); +lean_inc(x_35); +x_100 = l_Lean_addMacroScope(x_35, x_99, x_13); x_101 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__8; x_102 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_14); +lean_ctor_set(x_102, 1, x_31); x_103 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__9; -lean_inc(x_18); +lean_inc(x_33); x_104 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_18); +lean_ctor_set(x_104, 1, x_33); x_105 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_105, 0, x_102); lean_ctor_set(x_105, 1, x_104); -lean_inc(x_23); +lean_inc(x_19); x_106 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_106, 0, x_23); +lean_ctor_set(x_106, 0, x_19); lean_ctor_set(x_106, 1, x_98); lean_ctor_set(x_106, 2, x_100); lean_ctor_set(x_106, 3, x_105); -lean_inc(x_23); -x_107 = l_Lean_Syntax_node2(x_23, x_30, x_35, x_106); -lean_inc(x_39); -lean_inc(x_23); -x_108 = l_Lean_Syntax_node1(x_23, x_39, x_107); -lean_inc(x_38); -lean_inc(x_23); -x_109 = l_Lean_Syntax_node2(x_23, x_59, x_38, x_108); +lean_inc(x_19); +x_107 = l_Lean_Syntax_node2(x_19, x_23, x_40, x_106); +lean_inc(x_24); +lean_inc(x_19); +x_108 = l_Lean_Syntax_node1(x_19, x_24, x_107); +lean_inc(x_32); +lean_inc(x_19); +x_109 = l_Lean_Syntax_node2(x_19, x_59, x_32, x_108); x_110 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__10; -x_111 = l_Lean_Name_mkStr4(x_28, x_29, x_40, x_110); +x_111 = l_Lean_Name_mkStr4(x_16, x_37, x_15, x_110); x_112 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__11; -lean_inc(x_23); +lean_inc(x_19); x_113 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_113, 0, x_23); +lean_ctor_set(x_113, 0, x_19); lean_ctor_set(x_113, 1, x_112); x_114 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__13; x_115 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__14; -x_116 = l_Lean_addMacroScope(x_32, x_115, x_15); -lean_inc(x_23); +x_116 = l_Lean_addMacroScope(x_35, x_115, x_13); +lean_inc(x_19); x_117 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_117, 0, x_23); +lean_ctor_set(x_117, 0, x_19); lean_ctor_set(x_117, 1, x_114); lean_ctor_set(x_117, 2, x_116); -lean_ctor_set(x_117, 3, x_18); -lean_inc(x_23); -x_118 = l_Lean_Syntax_node3(x_23, x_111, x_34, x_113, x_117); -lean_inc(x_38); -lean_inc(x_23); -x_119 = l_Lean_Syntax_node4(x_23, x_26, x_33, x_118, x_25, x_38); -lean_inc(x_23); -x_120 = l_Lean_Syntax_node5(x_23, x_46, x_48, x_97, x_109, x_119, x_38); -lean_inc(x_23); -x_121 = l_Lean_Syntax_node2(x_23, x_13, x_92, x_120); -x_122 = l_Lean_Syntax_node4(x_23, x_39, x_16, x_37, x_80, x_121); +lean_ctor_set(x_117, 3, x_33); +lean_inc(x_19); +x_118 = l_Lean_Syntax_node3(x_19, x_111, x_17, x_113, x_117); +lean_inc(x_32); +lean_inc(x_19); +x_119 = l_Lean_Syntax_node4(x_19, x_30, x_18, x_118, x_20, x_32); +lean_inc(x_19); +x_120 = l_Lean_Syntax_node5(x_19, x_46, x_48, x_97, x_109, x_119, x_32); +lean_inc(x_19); +x_121 = l_Lean_Syntax_node2(x_19, x_38, x_92, x_120); +x_122 = l_Lean_Syntax_node4(x_19, x_24, x_34, x_22, x_80, x_121); x_123 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_17); +lean_ctor_set(x_123, 1, x_29); return x_123; } block_234: { 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_inc_ref(x_134); -x_156 = l_Array_append___redArg(x_134, x_155); +lean_inc_ref(x_149); +x_156 = l_Array_append___redArg(x_149, x_155); lean_dec_ref(x_155); -lean_inc(x_152); -lean_inc(x_132); +lean_inc(x_137); +lean_inc(x_131); x_157 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_157, 0, x_132); -lean_ctor_set(x_157, 1, x_152); +lean_ctor_set(x_157, 0, x_131); +lean_ctor_set(x_157, 1, x_137); lean_ctor_set(x_157, 2, x_156); -lean_inc(x_135); -lean_inc(x_145); -lean_inc(x_136); -lean_inc(x_132); -x_158 = l_Lean_Syntax_node4(x_132, x_136, x_145, x_126, x_135, x_157); -lean_inc(x_132); -x_159 = l_Lean_Syntax_node4(x_132, x_150, x_153, x_140, x_138, x_158); -lean_inc_n(x_151, 2); -lean_inc(x_132); -x_160 = l_Lean_Syntax_node4(x_132, x_137, x_151, x_151, x_144, x_159); +lean_inc(x_134); +lean_inc(x_129); +lean_inc(x_143); +lean_inc(x_131); +x_158 = l_Lean_Syntax_node4(x_131, x_143, x_129, x_154, x_134, x_157); +lean_inc(x_131); +x_159 = l_Lean_Syntax_node4(x_131, x_152, x_148, x_135, x_130, x_158); +lean_inc_n(x_145, 2); +lean_inc(x_131); +x_160 = l_Lean_Syntax_node4(x_131, x_132, x_145, x_145, x_139, x_159); x_161 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__27; x_162 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__28; -lean_inc(x_132); +lean_inc(x_131); x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_132); +lean_ctor_set(x_163, 0, x_131); lean_ctor_set(x_163, 1, x_162); x_164 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__30; x_165 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__31; -lean_inc(x_127); -lean_inc(x_146); -x_166 = l_Lean_addMacroScope(x_146, x_165, x_127); -x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__32; lean_inc(x_125); +lean_inc(x_147); +x_166 = l_Lean_addMacroScope(x_147, x_165, x_125); +x_167 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__32; +lean_inc(x_144); x_168 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_168, 0, x_167); -lean_ctor_set(x_168, 1, x_125); -lean_inc(x_129); +lean_ctor_set(x_168, 1, x_144); +lean_inc(x_146); x_169 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_169, 0, x_168); -lean_ctor_set(x_169, 1, x_129); -lean_inc(x_132); +lean_ctor_set(x_169, 1, x_146); +lean_inc(x_131); x_170 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_170, 0, x_132); +lean_ctor_set(x_170, 0, x_131); lean_ctor_set(x_170, 1, x_164); lean_ctor_set(x_170, 2, x_166); lean_ctor_set(x_170, 3, x_169); x_171 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__35; -lean_inc_ref(x_154); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_172 = l_Lean_Name_mkStr4(x_139, x_141, x_154, x_171); +lean_inc_ref(x_126); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_172 = l_Lean_Name_mkStr4(x_127, x_151, x_126, x_171); x_173 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__22; -lean_inc_ref(x_154); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_174 = l_Lean_Name_mkStr4(x_139, x_141, x_154, x_173); +lean_inc_ref(x_126); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_174 = l_Lean_Name_mkStr4(x_127, x_151, x_126, x_173); x_175 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__23; -lean_inc(x_132); +lean_inc(x_131); x_176 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_176, 0, x_132); +lean_ctor_set(x_176, 0, x_131); lean_ctor_set(x_176, 1, x_175); x_177 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__25; x_178 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__27; x_179 = lean_box(0); -lean_inc(x_127); -lean_inc(x_146); -x_180 = l_Lean_addMacroScope(x_146, x_179, x_127); +lean_inc(x_125); +lean_inc(x_147); +x_180 = l_Lean_addMacroScope(x_147, x_179, x_125); x_181 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__29; -lean_inc_ref(x_130); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_182 = l_Lean_Name_mkStr3(x_139, x_141, x_130); +lean_inc_ref(x_138); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_182 = l_Lean_Name_mkStr3(x_127, x_151, x_138); x_183 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_183, 0, x_182); x_184 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__30; -lean_inc_ref(x_130); -lean_inc_ref(x_139); -x_185 = l_Lean_Name_mkStr3(x_139, x_184, x_130); +lean_inc_ref(x_138); +lean_inc_ref(x_127); +x_185 = l_Lean_Name_mkStr3(x_127, x_184, x_138); x_186 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_186, 0, x_185); -lean_inc_ref(x_139); -x_187 = l_Lean_Name_mkStr2(x_139, x_184); +lean_inc_ref(x_127); +x_187 = l_Lean_Name_mkStr2(x_127, x_184); x_188 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_188, 0, x_187); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_189 = l_Lean_Name_mkStr2(x_139, x_141); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_189 = l_Lean_Name_mkStr2(x_127, x_151); x_190 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_190, 0, x_189); -lean_inc_ref(x_139); -x_191 = l_Lean_Name_mkStr1(x_139); +lean_inc_ref(x_127); +x_191 = l_Lean_Name_mkStr1(x_127); x_192 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_192, 0, x_191); -lean_inc(x_129); +lean_inc(x_146); x_193 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_193, 0, x_192); -lean_ctor_set(x_193, 1, x_129); +lean_ctor_set(x_193, 1, x_146); x_194 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_194, 0, x_190); lean_ctor_set(x_194, 1, x_193); @@ -23171,166 +23171,166 @@ lean_ctor_set(x_197, 1, x_196); x_198 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_198, 0, x_181); lean_ctor_set(x_198, 1, x_197); -lean_inc(x_132); +lean_inc(x_131); x_199 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_199, 0, x_132); +lean_ctor_set(x_199, 0, x_131); lean_ctor_set(x_199, 1, x_178); lean_ctor_set(x_199, 2, x_180); lean_ctor_set(x_199, 3, x_198); -lean_inc(x_132); -x_200 = l_Lean_Syntax_node1(x_132, x_177, x_199); -lean_inc(x_132); -x_201 = l_Lean_Syntax_node2(x_132, x_174, x_176, x_200); +lean_inc(x_131); +x_200 = l_Lean_Syntax_node1(x_131, x_177, x_199); +lean_inc(x_131); +x_201 = l_Lean_Syntax_node2(x_131, x_174, x_176, x_200); x_202 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__37; x_203 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__38; -lean_inc(x_132); +lean_inc(x_131); x_204 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_204, 0, x_132); +lean_ctor_set(x_204, 0, x_131); lean_ctor_set(x_204, 1, x_203); -lean_inc(x_132); -x_205 = l_Lean_Syntax_node1(x_132, x_202, x_204); +lean_inc(x_131); +x_205 = l_Lean_Syntax_node1(x_131, x_202, x_204); x_206 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__7; -lean_inc(x_132); +lean_inc(x_131); x_207 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_207, 0, x_132); +lean_ctor_set(x_207, 0, x_131); lean_ctor_set(x_207, 1, x_206); +lean_inc(x_140); +lean_inc(x_137); lean_inc(x_131); -lean_inc(x_152); -lean_inc(x_132); -x_208 = l_Lean_Syntax_node1(x_132, x_152, x_131); +x_208 = l_Lean_Syntax_node1(x_131, x_137, x_140); lean_inc(x_205); -lean_inc(x_152); -lean_inc(x_132); -x_209 = l_Lean_Syntax_node3(x_132, x_152, x_205, x_207, x_208); +lean_inc(x_137); +lean_inc(x_131); +x_209 = l_Lean_Syntax_node3(x_131, x_137, x_205, x_207, x_208); x_210 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__34; -lean_inc(x_132); +lean_inc(x_131); x_211 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_211, 0, x_132); +lean_ctor_set(x_211, 0, x_131); lean_ctor_set(x_211, 1, x_210); -lean_inc(x_132); -x_212 = l_Lean_Syntax_node3(x_132, x_172, x_201, x_209, x_211); +lean_inc(x_131); +x_212 = l_Lean_Syntax_node3(x_131, x_172, x_201, x_209, x_211); x_213 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__15; -lean_inc_ref(x_154); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_214 = l_Lean_Name_mkStr4(x_139, x_141, x_154, x_213); +lean_inc_ref(x_126); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_214 = l_Lean_Name_mkStr4(x_127, x_151, x_126, x_213); x_215 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__5; x_216 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__6; -lean_inc(x_127); -lean_inc(x_146); -x_217 = l_Lean_addMacroScope(x_146, x_216, x_127); -x_218 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__7; lean_inc(x_125); +lean_inc(x_147); +x_217 = l_Lean_addMacroScope(x_147, x_216, x_125); +x_218 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__7; +lean_inc(x_144); x_219 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_219, 0, x_218); -lean_ctor_set(x_219, 1, x_125); +lean_ctor_set(x_219, 1, x_144); x_220 = l___private_Lake_DSL_Targets_0__Lake_DSL_mkConfigDeclDef___closed__9; -lean_inc(x_129); +lean_inc(x_146); x_221 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_221, 0, x_220); -lean_ctor_set(x_221, 1, x_129); +lean_ctor_set(x_221, 1, x_146); x_222 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_222, 0, x_219); lean_ctor_set(x_222, 1, x_221); -lean_inc(x_132); +lean_inc(x_131); x_223 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_223, 0, x_132); +lean_ctor_set(x_223, 0, x_131); lean_ctor_set(x_223, 1, x_215); lean_ctor_set(x_223, 2, x_217); lean_ctor_set(x_223, 3, x_222); -lean_inc(x_152); -lean_inc(x_132); -x_224 = l_Lean_Syntax_node1(x_132, x_152, x_142); +lean_inc(x_137); +lean_inc(x_131); +x_224 = l_Lean_Syntax_node1(x_131, x_137, x_141); lean_inc(x_214); -lean_inc(x_132); -x_225 = l_Lean_Syntax_node2(x_132, x_214, x_223, x_224); +lean_inc(x_131); +x_225 = l_Lean_Syntax_node2(x_131, x_214, x_223, x_224); +lean_inc(x_129); +lean_inc(x_153); +lean_inc(x_128); lean_inc(x_145); -lean_inc(x_149); -lean_inc(x_147); -lean_inc(x_151); -lean_inc(x_132); -x_226 = l_Lean_Syntax_node8(x_132, x_161, x_151, x_163, x_147, x_149, x_170, x_212, x_145, x_225); +lean_inc(x_131); +x_226 = l_Lean_Syntax_node8(x_131, x_161, x_145, x_163, x_128, x_153, x_170, x_212, x_129, x_225); x_227 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__40; -lean_inc_ref(x_130); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_228 = l_Lean_Name_mkStr4(x_139, x_141, x_130, x_227); +lean_inc_ref(x_138); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_228 = l_Lean_Name_mkStr4(x_127, x_151, x_138, x_227); x_229 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__41; -lean_inc_ref(x_130); -lean_inc_ref(x_141); -lean_inc_ref(x_139); -x_230 = l_Lean_Name_mkStr4(x_139, x_141, x_130, x_229); -if (lean_obj_tag(x_133) == 1) +lean_inc_ref(x_138); +lean_inc_ref(x_151); +lean_inc_ref(x_127); +x_230 = l_Lean_Name_mkStr4(x_127, x_151, x_138, x_229); +if (lean_obj_tag(x_150) == 1) { lean_object* x_231; lean_object* x_232; -x_231 = lean_ctor_get(x_133, 0); +x_231 = lean_ctor_get(x_150, 0); lean_inc(x_231); -lean_dec_ref(x_133); +lean_dec_ref(x_150); x_232 = l_Array_mkArray1___redArg(x_231); -x_13 = x_228; -x_14 = x_125; -x_15 = x_127; -x_16 = x_160; +x_13 = x_125; +x_14 = x_205; +x_15 = x_126; +x_16 = x_127; x_17 = x_128; x_18 = x_129; -x_19 = x_130; -x_20 = x_205; -x_21 = x_131; -x_22 = x_214; -x_23 = x_132; -x_24 = x_134; -x_25 = x_135; -x_26 = x_136; -x_27 = x_206; -x_28 = x_139; -x_29 = x_141; +x_19 = x_131; +x_20 = x_134; +x_21 = x_133; +x_22 = x_226; +x_23 = x_136; +x_24 = x_137; +x_25 = x_138; +x_26 = x_206; +x_27 = x_140; +x_28 = x_214; +x_29 = x_142; x_30 = x_143; -x_31 = x_230; -x_32 = x_146; -x_33 = x_145; -x_34 = x_147; -x_35 = x_149; -x_36 = x_148; -x_37 = x_226; -x_38 = x_151; -x_39 = x_152; -x_40 = x_154; +x_31 = x_144; +x_32 = x_145; +x_33 = x_146; +x_34 = x_160; +x_35 = x_147; +x_36 = x_149; +x_37 = x_151; +x_38 = x_228; +x_39 = x_230; +x_40 = x_153; x_41 = x_232; goto block_124; } else { lean_object* x_233; -lean_dec(x_133); +lean_dec(x_150); x_233 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_13 = x_228; -x_14 = x_125; -x_15 = x_127; -x_16 = x_160; +x_13 = x_125; +x_14 = x_205; +x_15 = x_126; +x_16 = x_127; x_17 = x_128; x_18 = x_129; -x_19 = x_130; -x_20 = x_205; -x_21 = x_131; -x_22 = x_214; -x_23 = x_132; -x_24 = x_134; -x_25 = x_135; -x_26 = x_136; -x_27 = x_206; -x_28 = x_139; -x_29 = x_141; +x_19 = x_131; +x_20 = x_134; +x_21 = x_133; +x_22 = x_226; +x_23 = x_136; +x_24 = x_137; +x_25 = x_138; +x_26 = x_206; +x_27 = x_140; +x_28 = x_214; +x_29 = x_142; x_30 = x_143; -x_31 = x_230; -x_32 = x_146; -x_33 = x_145; -x_34 = x_147; -x_35 = x_149; -x_36 = x_148; -x_37 = x_226; -x_38 = x_151; -x_39 = x_152; -x_40 = x_154; +x_31 = x_144; +x_32 = x_145; +x_33 = x_146; +x_34 = x_160; +x_35 = x_147; +x_36 = x_149; +x_37 = x_151; +x_38 = x_228; +x_39 = x_230; +x_40 = x_153; x_41 = x_233; goto block_124; } @@ -23338,129 +23338,129 @@ goto block_124; block_281: { 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_inc_ref(x_245); -x_261 = l_Array_append___redArg(x_245, x_260); +lean_inc_ref(x_255); +x_261 = l_Array_append___redArg(x_255, x_260); lean_dec_ref(x_260); -lean_inc(x_257); -lean_inc(x_242); +lean_inc(x_243); +lean_inc(x_240); x_262 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_262, 0, x_242); -lean_ctor_set(x_262, 1, x_257); +lean_ctor_set(x_262, 0, x_240); +lean_ctor_set(x_262, 1, x_243); lean_ctor_set(x_262, 2, x_261); x_263 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__57; -lean_inc_ref(x_258); -lean_inc_ref(x_249); -lean_inc_ref(x_248); -x_264 = l_Lean_Name_mkStr4(x_248, x_249, x_258, x_263); +lean_inc_ref(x_236); +lean_inc_ref(x_256); +lean_inc_ref(x_237); +x_264 = l_Lean_Name_mkStr4(x_237, x_256, x_236, x_263); x_265 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__39; -lean_inc(x_242); +lean_inc(x_240); x_266 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_266, 0, x_242); +lean_ctor_set(x_266, 0, x_240); lean_ctor_set(x_266, 1, x_265); x_267 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__12; x_268 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__13; -lean_inc(x_237); -lean_inc(x_252); -x_269 = l_Lean_addMacroScope(x_252, x_268, x_237); +lean_inc(x_235); +lean_inc(x_253); +x_269 = l_Lean_addMacroScope(x_253, x_268, x_235); x_270 = lean_box(0); x_271 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___closed__16; -lean_inc(x_239); +lean_inc(x_252); x_272 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_272, 0, x_271); -lean_ctor_set(x_272, 1, x_239); -lean_inc(x_242); +lean_ctor_set(x_272, 1, x_252); +lean_inc(x_240); x_273 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_273, 0, x_242); +lean_ctor_set(x_273, 0, x_240); lean_ctor_set(x_273, 1, x_267); lean_ctor_set(x_273, 2, x_269); lean_ctor_set(x_273, 3, x_272); lean_inc_ref(x_266); lean_inc(x_264); -lean_inc(x_242); -x_274 = l_Lean_Syntax_node2(x_242, x_264, x_266, x_273); +lean_inc(x_240); +x_274 = l_Lean_Syntax_node2(x_240, x_264, x_266, x_273); x_275 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__14; -lean_inc(x_242); +lean_inc(x_240); x_276 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_276, 0, x_242); +lean_ctor_set(x_276, 0, x_240); lean_ctor_set(x_276, 1, x_275); -lean_inc_n(x_256, 2); -lean_inc(x_242); -x_277 = l_Lean_Syntax_node2(x_242, x_235, x_256, x_256); -if (lean_obj_tag(x_243) == 1) +lean_inc_n(x_251, 2); +lean_inc(x_240); +x_277 = l_Lean_Syntax_node2(x_240, x_239, x_251, x_251); +if (lean_obj_tag(x_250) == 1) { lean_object* x_278; lean_object* x_279; -x_278 = lean_ctor_get(x_243, 0); +x_278 = lean_ctor_get(x_250, 0); lean_inc(x_278); -lean_dec_ref(x_243); +lean_dec_ref(x_250); x_279 = l_Array_mkArray1___redArg(x_278); -x_125 = x_270; +x_125 = x_235; x_126 = x_236; x_127 = x_237; x_128 = x_238; -x_129 = x_239; -x_130 = x_240; -x_131 = x_241; -x_132 = x_242; -x_133 = x_244; -x_134 = x_245; -x_135 = x_277; -x_136 = x_246; -x_137 = x_247; -x_138 = x_274; -x_139 = x_248; -x_140 = x_262; -x_141 = x_249; -x_142 = x_250; -x_143 = x_264; -x_144 = x_251; -x_145 = x_276; +x_129 = x_276; +x_130 = x_274; +x_131 = x_240; +x_132 = x_241; +x_133 = x_242; +x_134 = x_277; +x_135 = x_262; +x_136 = x_264; +x_137 = x_243; +x_138 = x_244; +x_139 = x_245; +x_140 = x_246; +x_141 = x_247; +x_142 = x_248; +x_143 = x_249; +x_144 = x_270; +x_145 = x_251; x_146 = x_252; x_147 = x_253; x_148 = x_254; -x_149 = x_266; -x_150 = x_255; +x_149 = x_255; +x_150 = x_257; x_151 = x_256; -x_152 = x_257; -x_153 = x_259; -x_154 = x_258; +x_152 = x_258; +x_153 = x_266; +x_154 = x_259; x_155 = x_279; goto block_234; } else { lean_object* x_280; -lean_dec(x_243); +lean_dec(x_250); x_280 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_125 = x_270; +x_125 = x_235; x_126 = x_236; x_127 = x_237; x_128 = x_238; -x_129 = x_239; -x_130 = x_240; -x_131 = x_241; -x_132 = x_242; -x_133 = x_244; -x_134 = x_245; -x_135 = x_277; -x_136 = x_246; -x_137 = x_247; -x_138 = x_274; -x_139 = x_248; -x_140 = x_262; -x_141 = x_249; -x_142 = x_250; -x_143 = x_264; -x_144 = x_251; -x_145 = x_276; +x_129 = x_276; +x_130 = x_274; +x_131 = x_240; +x_132 = x_241; +x_133 = x_242; +x_134 = x_277; +x_135 = x_262; +x_136 = x_264; +x_137 = x_243; +x_138 = x_244; +x_139 = x_245; +x_140 = x_246; +x_141 = x_247; +x_142 = x_248; +x_143 = x_249; +x_144 = x_270; +x_145 = x_251; x_146 = x_252; x_147 = x_253; x_148 = x_254; -x_149 = x_266; -x_150 = x_255; +x_149 = x_255; +x_150 = x_257; x_151 = x_256; -x_152 = x_257; -x_153 = x_259; -x_154 = x_258; +x_152 = x_258; +x_153 = x_266; +x_154 = x_259; x_155 = x_280; goto block_234; } @@ -23469,93 +23469,93 @@ goto block_234; { uint8_t 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; x_306 = 0; -x_307 = l_Lean_mkIdentFrom(x_298, x_305, x_306); -lean_inc(x_298); -x_308 = l_Lake_Name_quoteFrom(x_298, x_284, x_306); +x_307 = l_Lean_mkIdentFrom(x_286, x_305, x_306); +lean_inc(x_286); +x_308 = l_Lake_Name_quoteFrom(x_286, x_288, x_306); x_309 = l_Lake_ExternLib_keyword; x_310 = l_Lake_Name_quoteFrom(x_282, x_309, x_306); -x_311 = l_Lean_SourceInfo_fromRef(x_283, x_306); -lean_dec(x_283); +x_311 = l_Lean_SourceInfo_fromRef(x_299, x_306); +lean_dec(x_299); x_312 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__16; -lean_inc_ref(x_302); +lean_inc_ref(x_295); lean_inc(x_301); lean_inc(x_311); x_313 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_313, 0, x_311); lean_ctor_set(x_313, 1, x_301); -lean_ctor_set(x_313, 2, x_302); +lean_ctor_set(x_313, 2, x_295); lean_inc(x_311); x_314 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_314, 0, x_311); -lean_ctor_set(x_314, 1, x_289); +lean_ctor_set(x_314, 1, x_300); x_315 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__68; lean_inc(x_311); -x_316 = l_Lean_Syntax_node1(x_311, x_292, x_307); -if (lean_obj_tag(x_285) == 1) +x_316 = l_Lean_Syntax_node1(x_311, x_294, x_307); +if (lean_obj_tag(x_302) == 1) { lean_object* x_317; lean_object* x_318; -x_317 = lean_ctor_get(x_285, 0); +x_317 = lean_ctor_get(x_302, 0); lean_inc(x_317); -lean_dec_ref(x_285); +lean_dec_ref(x_302); x_318 = l_Array_mkArray1___redArg(x_317); -x_235 = x_286; -x_236 = x_287; -x_237 = x_288; -x_238 = x_290; -x_239 = x_294; -x_240 = x_295; -x_241 = x_308; -x_242 = x_311; -x_243 = x_296; -x_244 = x_300; -x_245 = x_302; -x_246 = x_304; -x_247 = x_312; +x_235 = x_283; +x_236 = x_284; +x_237 = x_285; +x_238 = x_286; +x_239 = x_287; +x_240 = x_311; +x_241 = x_312; +x_242 = x_296; +x_243 = x_301; +x_244 = x_304; +x_245 = x_314; +x_246 = x_308; +x_247 = x_310; x_248 = x_291; -x_249 = x_293; -x_250 = x_310; -x_251 = x_314; -x_252 = x_297; -x_253 = x_298; -x_254 = x_299; -x_255 = x_315; -x_256 = x_313; -x_257 = x_301; -x_258 = x_303; -x_259 = x_316; +x_249 = x_290; +x_250 = x_289; +x_251 = x_313; +x_252 = x_292; +x_253 = x_293; +x_254 = x_316; +x_255 = x_295; +x_256 = x_298; +x_257 = x_297; +x_258 = x_315; +x_259 = x_303; x_260 = x_318; goto block_281; } else { lean_object* x_319; -lean_dec(x_285); +lean_dec(x_302); x_319 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__35; -x_235 = x_286; -x_236 = x_287; -x_237 = x_288; -x_238 = x_290; -x_239 = x_294; -x_240 = x_295; -x_241 = x_308; -x_242 = x_311; -x_243 = x_296; -x_244 = x_300; -x_245 = x_302; -x_246 = x_304; -x_247 = x_312; +x_235 = x_283; +x_236 = x_284; +x_237 = x_285; +x_238 = x_286; +x_239 = x_287; +x_240 = x_311; +x_241 = x_312; +x_242 = x_296; +x_243 = x_301; +x_244 = x_304; +x_245 = x_314; +x_246 = x_308; +x_247 = x_310; x_248 = x_291; -x_249 = x_293; -x_250 = x_310; -x_251 = x_314; -x_252 = x_297; -x_253 = x_298; -x_254 = x_299; -x_255 = x_315; -x_256 = x_313; -x_257 = x_301; -x_258 = x_303; -x_259 = x_316; +x_249 = x_290; +x_250 = x_289; +x_251 = x_313; +x_252 = x_292; +x_253 = x_293; +x_254 = x_316; +x_255 = x_295; +x_256 = x_298; +x_257 = x_297; +x_258 = x_315; +x_259 = x_303; x_260 = x_319; goto block_281; } @@ -23592,13 +23592,13 @@ lean_dec_ref(x_342); x_345 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__41; x_346 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_347 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__42; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_348 = l_Lean_Name_mkStr4(x_329, x_321, x_346, x_347); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_348 = l_Lean_Name_mkStr4(x_322, x_325, x_346, x_347); x_349 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__43; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_350 = l_Lean_Name_mkStr4(x_329, x_321, x_346, x_349); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_350 = l_Lean_Name_mkStr4(x_322, x_325, x_346, x_349); x_351 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_352 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; lean_inc(x_340); @@ -23612,9 +23612,9 @@ lean_inc(x_340); x_354 = l_Lean_Syntax_node1(x_340, x_350, x_353); x_355 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__47; x_356 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__48; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_357 = l_Lean_Name_mkStr4(x_329, x_321, x_355, x_356); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_357 = l_Lean_Name_mkStr4(x_322, x_325, x_355, x_356); x_358 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_359 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__24; x_360 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; @@ -23658,10 +23658,10 @@ x_373 = l_Lean_Syntax_node2(x_343, x_348, x_367, x_372); x_374 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_375 = lean_array_push(x_374, x_365); x_376 = lean_array_push(x_375, x_373); -x_377 = l_Lake_DSL_expandAttrs(x_326); +x_377 = l_Lake_DSL_expandAttrs(x_321); x_378 = l_Array_append___redArg(x_376, x_377); lean_dec_ref(x_377); -x_379 = l_Lake_DSL_expandIdentOrStrAsIdent(x_324); +x_379 = l_Lake_DSL_expandIdentOrStrAsIdent(x_327); x_380 = l_Lean_TSyntax_getId(x_379); x_381 = l_Lean_Name_hasMacroScopes(x_380); if (x_381 == 0) @@ -23669,28 +23669,28 @@ if (x_381 == 0) lean_object* x_382; lean_inc(x_380); x_382 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___lam__1(x_380); -x_283 = x_338; -x_284 = x_380; -x_285 = x_323; -x_286 = x_325; -x_287 = x_327; -x_288 = x_336; -x_289 = x_359; -x_290 = x_344; -x_291 = x_329; -x_292 = x_345; -x_293 = x_321; -x_294 = x_362; -x_295 = x_322; -x_296 = x_331; -x_297 = x_335; -x_298 = x_379; -x_299 = x_378; -x_300 = x_328; +x_283 = x_336; +x_284 = x_346; +x_285 = x_322; +x_286 = x_379; +x_287 = x_323; +x_288 = x_380; +x_289 = x_331; +x_290 = x_326; +x_291 = x_344; +x_292 = x_362; +x_293 = x_335; +x_294 = x_345; +x_295 = x_352; +x_296 = x_378; +x_297 = x_324; +x_298 = x_325; +x_299 = x_338; +x_300 = x_359; x_301 = x_351; -x_302 = x_352; -x_303 = x_346; -x_304 = x_330; +x_302 = x_330; +x_303 = x_329; +x_304 = x_328; x_305 = x_382; goto block_320; } @@ -23707,28 +23707,28 @@ x_385 = lean_ctor_get(x_383, 0); x_386 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___lam__1(x_385); lean_ctor_set(x_383, 0, x_386); x_387 = l_Lean_MacroScopesView_review(x_383); -x_283 = x_338; -x_284 = x_380; -x_285 = x_323; -x_286 = x_325; -x_287 = x_327; -x_288 = x_336; -x_289 = x_359; -x_290 = x_344; -x_291 = x_329; -x_292 = x_345; -x_293 = x_321; -x_294 = x_362; -x_295 = x_322; -x_296 = x_331; -x_297 = x_335; -x_298 = x_379; -x_299 = x_378; -x_300 = x_328; +x_283 = x_336; +x_284 = x_346; +x_285 = x_322; +x_286 = x_379; +x_287 = x_323; +x_288 = x_380; +x_289 = x_331; +x_290 = x_326; +x_291 = x_344; +x_292 = x_362; +x_293 = x_335; +x_294 = x_345; +x_295 = x_352; +x_296 = x_378; +x_297 = x_324; +x_298 = x_325; +x_299 = x_338; +x_300 = x_359; x_301 = x_351; -x_302 = x_352; -x_303 = x_346; -x_304 = x_330; +x_302 = x_330; +x_303 = x_329; +x_304 = x_328; x_305 = x_387; goto block_320; } @@ -23751,28 +23751,28 @@ lean_ctor_set(x_393, 1, x_389); lean_ctor_set(x_393, 2, x_390); lean_ctor_set(x_393, 3, x_391); x_394 = l_Lean_MacroScopesView_review(x_393); -x_283 = x_338; -x_284 = x_380; -x_285 = x_323; -x_286 = x_325; -x_287 = x_327; -x_288 = x_336; -x_289 = x_359; -x_290 = x_344; -x_291 = x_329; -x_292 = x_345; -x_293 = x_321; -x_294 = x_362; -x_295 = x_322; -x_296 = x_331; -x_297 = x_335; -x_298 = x_379; -x_299 = x_378; -x_300 = x_328; +x_283 = x_336; +x_284 = x_346; +x_285 = x_322; +x_286 = x_379; +x_287 = x_323; +x_288 = x_380; +x_289 = x_331; +x_290 = x_326; +x_291 = x_344; +x_292 = x_362; +x_293 = x_335; +x_294 = x_345; +x_295 = x_352; +x_296 = x_378; +x_297 = x_324; +x_298 = x_325; +x_299 = x_338; +x_300 = x_359; x_301 = x_351; -x_302 = x_352; -x_303 = x_346; -x_304 = x_330; +x_302 = x_330; +x_303 = x_329; +x_304 = x_328; x_305 = x_394; goto block_320; } @@ -23822,13 +23822,13 @@ lean_dec_ref(x_406); x_409 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__41; x_410 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__56; x_411 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__42; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_412 = l_Lean_Name_mkStr4(x_329, x_321, x_410, x_411); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_412 = l_Lean_Name_mkStr4(x_322, x_325, x_410, x_411); x_413 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__43; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_414 = l_Lean_Name_mkStr4(x_329, x_321, x_410, x_413); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_414 = l_Lean_Name_mkStr4(x_322, x_325, x_410, x_413); x_415 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__45; x_416 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__46; lean_inc(x_404); @@ -23842,9 +23842,9 @@ lean_inc(x_404); x_418 = l_Lean_Syntax_node1(x_404, x_414, x_417); x_419 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__47; x_420 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__48; -lean_inc_ref(x_321); -lean_inc_ref(x_329); -x_421 = l_Lean_Name_mkStr4(x_329, x_321, x_419, x_420); +lean_inc_ref(x_325); +lean_inc_ref(x_322); +x_421 = l_Lean_Name_mkStr4(x_322, x_325, x_419, x_420); x_422 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__23; x_423 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__24; x_424 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandTargetCommand___closed__25; @@ -23888,10 +23888,10 @@ x_437 = l_Lean_Syntax_node2(x_407, x_412, x_431, x_436); x_438 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandModuleFacetDecl___closed__12; x_439 = lean_array_push(x_438, x_429); x_440 = lean_array_push(x_439, x_437); -x_441 = l_Lake_DSL_expandAttrs(x_326); +x_441 = l_Lake_DSL_expandAttrs(x_321); x_442 = l_Array_append___redArg(x_440, x_441); lean_dec_ref(x_441); -x_443 = l_Lake_DSL_expandIdentOrStrAsIdent(x_324); +x_443 = l_Lake_DSL_expandIdentOrStrAsIdent(x_327); x_444 = l_Lean_TSyntax_getId(x_443); x_445 = l_Lean_Name_hasMacroScopes(x_444); if (x_445 == 0) @@ -23899,28 +23899,28 @@ if (x_445 == 0) lean_object* x_446; lean_inc(x_444); x_446 = l___private_Lake_DSL_Targets_0__Lake_DSL_expandExternLibCommand___lam__1(x_444); -x_283 = x_401; -x_284 = x_444; -x_285 = x_323; -x_286 = x_325; -x_287 = x_327; -x_288 = x_397; -x_289 = x_423; -x_290 = x_408; -x_291 = x_329; -x_292 = x_409; -x_293 = x_321; -x_294 = x_426; -x_295 = x_322; -x_296 = x_331; -x_297 = x_396; -x_298 = x_443; -x_299 = x_442; -x_300 = x_328; +x_283 = x_397; +x_284 = x_410; +x_285 = x_322; +x_286 = x_443; +x_287 = x_323; +x_288 = x_444; +x_289 = x_331; +x_290 = x_326; +x_291 = x_408; +x_292 = x_426; +x_293 = x_396; +x_294 = x_409; +x_295 = x_416; +x_296 = x_442; +x_297 = x_324; +x_298 = x_325; +x_299 = x_401; +x_300 = x_423; x_301 = x_415; -x_302 = x_416; -x_303 = x_410; -x_304 = x_330; +x_302 = x_330; +x_303 = x_329; +x_304 = x_328; x_305 = x_446; goto block_320; } @@ -23958,28 +23958,28 @@ lean_ctor_set(x_454, 1, x_449); lean_ctor_set(x_454, 2, x_450); lean_ctor_set(x_454, 3, x_451); x_455 = l_Lean_MacroScopesView_review(x_454); -x_283 = x_401; -x_284 = x_444; -x_285 = x_323; -x_286 = x_325; -x_287 = x_327; -x_288 = x_397; -x_289 = x_423; -x_290 = x_408; -x_291 = x_329; -x_292 = x_409; -x_293 = x_321; -x_294 = x_426; -x_295 = x_322; -x_296 = x_331; -x_297 = x_396; -x_298 = x_443; -x_299 = x_442; -x_300 = x_328; +x_283 = x_397; +x_284 = x_410; +x_285 = x_322; +x_286 = x_443; +x_287 = x_323; +x_288 = x_444; +x_289 = x_331; +x_290 = x_326; +x_291 = x_408; +x_292 = x_426; +x_293 = x_396; +x_294 = x_409; +x_295 = x_416; +x_296 = x_442; +x_297 = x_324; +x_298 = x_325; +x_299 = x_401; +x_300 = x_423; x_301 = x_415; -x_302 = x_416; -x_303 = x_410; -x_304 = x_330; +x_302 = x_330; +x_303 = x_329; +x_304 = x_328; x_305 = x_455; goto block_320; } @@ -24127,16 +24127,16 @@ lean_object* x_497; lean_dec(x_458); x_497 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_497, 0, x_492); -x_321 = x_467; -x_322 = x_468; -x_323 = x_462; -x_324 = x_459; -x_325 = x_474; -x_326 = x_460; -x_327 = x_486; -x_328 = x_461; -x_329 = x_466; -x_330 = x_469; +x_321 = x_459; +x_322 = x_466; +x_323 = x_474; +x_324 = x_460; +x_325 = x_467; +x_326 = x_469; +x_327 = x_461; +x_328 = x_468; +x_329 = x_486; +x_330 = x_462; x_331 = x_497; x_332 = x_463; x_333 = x_464; @@ -24150,16 +24150,16 @@ lean_object* x_498; lean_dec(x_487); lean_dec(x_458); x_498 = lean_box(0); -x_321 = x_467; -x_322 = x_468; -x_323 = x_462; -x_324 = x_459; -x_325 = x_474; -x_326 = x_460; -x_327 = x_486; -x_328 = x_461; -x_329 = x_466; -x_330 = x_469; +x_321 = x_459; +x_322 = x_466; +x_323 = x_474; +x_324 = x_460; +x_325 = x_467; +x_326 = x_469; +x_327 = x_461; +x_328 = x_468; +x_329 = x_486; +x_330 = x_462; x_331 = x_498; x_332 = x_463; x_333 = x_464; @@ -24217,9 +24217,9 @@ x_512 = l_Lean_Syntax_getArg(x_507, x_8); lean_dec(x_507); x_513 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_513, 0, x_512); -x_459 = x_506; -x_460 = x_501; -x_461 = x_502; +x_459 = x_501; +x_460 = x_502; +x_461 = x_506; x_462 = x_513; x_463 = x_2; x_464 = x_3; @@ -24231,9 +24231,9 @@ else lean_object* x_514; lean_dec(x_507); x_514 = lean_box(0); -x_459 = x_506; -x_460 = x_501; -x_461 = x_502; +x_459 = x_501; +x_460 = x_502; +x_461 = x_506; x_462 = x_514; x_463 = x_2; x_464 = x_3; diff --git a/stage0/stdlib/Lake/Util/Url.c b/stage0/stdlib/Lake/Util/Url.c index 909d297caeaf..9a38da8f28ef 100644 --- a/stage0/stdlib/Lake/Util/Url.c +++ b/stage0/stdlib/Lake/Util/Url.c @@ -1621,8 +1621,8 @@ x_16 = 3; x_17 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_17, 0, x_15); lean_ctor_set_uint8(x_17, sizeof(void*)*1, x_16); -x_18 = lean_array_push(x_10, x_17); -x_5 = x_11; +x_18 = lean_array_push(x_12, x_17); +x_5 = x_10; x_6 = x_18; x_7 = lean_box(0); goto block_9; @@ -1631,8 +1631,8 @@ goto block_9; { lean_object* x_23; lean_object* x_24; x_23 = l_Lake_getUrl_x3f___closed__2; -x_24 = lean_array_push(x_20, x_23); -x_5 = x_21; +x_24 = lean_array_push(x_22, x_23); +x_5 = x_20; x_6 = x_24; x_7 = lean_box(0); goto block_9; @@ -1647,8 +1647,8 @@ x_32 = 3; x_33 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_33, 0, x_31); lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); -x_34 = lean_array_push(x_26, x_33); -x_5 = x_27; +x_34 = lean_array_push(x_28, x_33); +x_5 = x_26; x_6 = x_34; x_7 = lean_box(0); goto block_9; @@ -1658,10 +1658,10 @@ goto block_9; if (lean_obj_tag(x_41) == 0) { lean_dec_ref(x_39); -lean_dec(x_38); -x_20 = x_36; -x_21 = x_37; -x_22 = lean_box(0); +lean_dec(x_36); +x_20 = x_37; +x_21 = lean_box(0); +x_22 = x_40; goto block_25; } else @@ -1678,7 +1678,7 @@ if (x_45 == 0) { lean_object* x_46; uint8_t x_47; lean_free_object(x_41); -lean_dec(x_38); +lean_dec(x_36); x_46 = lean_unsigned_to_nat(404u); x_47 = lean_nat_dec_eq(x_43, x_46); if (x_47 == 0) @@ -1699,7 +1699,7 @@ x_55 = 3; x_56 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_56, 0, x_54); lean_ctor_set_uint8(x_56, sizeof(void*)*1, x_55); -x_57 = lean_array_push(x_36, x_56); +x_57 = lean_array_push(x_40, x_56); x_5 = x_37; x_6 = x_57; x_7 = lean_box(0); @@ -1714,7 +1714,7 @@ lean_dec(x_37); x_58 = lean_box(0); x_59 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_36); +lean_ctor_set(x_59, 1, x_40); return x_59; } } @@ -1729,7 +1729,7 @@ lean_dec_ref(x_39); x_61 = lean_string_utf8_byte_size(x_60); x_62 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_38); +lean_ctor_set(x_62, 1, x_36); lean_ctor_set(x_62, 2, x_61); x_63 = l_String_Slice_trimAscii(x_62); lean_dec_ref(x_62); @@ -1747,7 +1747,7 @@ lean_dec_ref(x_64); lean_ctor_set(x_41, 0, x_67); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_41); -lean_ctor_set(x_68, 1, x_36); +lean_ctor_set(x_68, 1, x_40); return x_68; } } @@ -1762,7 +1762,7 @@ x_71 = lean_nat_dec_eq(x_69, x_70); if (x_71 == 0) { lean_object* x_72; uint8_t x_73; -lean_dec(x_38); +lean_dec(x_36); x_72 = lean_unsigned_to_nat(404u); x_73 = lean_nat_dec_eq(x_69, x_72); if (x_73 == 0) @@ -1783,7 +1783,7 @@ x_81 = 3; x_82 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_82, 0, x_80); lean_ctor_set_uint8(x_82, sizeof(void*)*1, x_81); -x_83 = lean_array_push(x_36, x_82); +x_83 = lean_array_push(x_40, x_82); x_5 = x_37; x_6 = x_83; x_7 = lean_box(0); @@ -1798,7 +1798,7 @@ lean_dec(x_37); x_84 = lean_box(0); x_85 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_36); +lean_ctor_set(x_85, 1, x_40); return x_85; } } @@ -1813,7 +1813,7 @@ lean_dec_ref(x_39); x_87 = lean_string_utf8_byte_size(x_86); x_88 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_38); +lean_ctor_set(x_88, 1, x_36); lean_ctor_set(x_88, 2, x_87); x_89 = l_String_Slice_trimAscii(x_88); lean_dec_ref(x_88); @@ -1832,7 +1832,7 @@ x_94 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_94, 0, x_93); x_95 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_36); +lean_ctor_set(x_95, 1, x_40); return x_95; } } @@ -1842,15 +1842,15 @@ return x_95; { lean_object* x_103; lean_object* x_104; x_103 = l_Lake_getUrl_x3f___closed__6; -x_104 = l_Lake_JsonObject_getJson_x3f(x_97, x_103); -lean_dec(x_97); +x_104 = l_Lake_JsonObject_getJson_x3f(x_100, x_103); +lean_dec(x_100); if (lean_obj_tag(x_104) == 0) { lean_dec_ref(x_101); -lean_dec(x_100); +lean_dec(x_97); x_20 = x_98; -x_21 = x_99; -x_22 = lean_box(0); +x_21 = lean_box(0); +x_22 = x_102; goto block_25; } else @@ -1864,7 +1864,7 @@ if (lean_obj_tag(x_106) == 0) { lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_dec_ref(x_101); -lean_dec(x_100); +lean_dec(x_97); x_107 = lean_ctor_get(x_106, 0); lean_inc(x_107); lean_dec_ref(x_106); @@ -1872,8 +1872,8 @@ x_108 = l_Lake_getUrl_x3f___closed__7; x_109 = lean_string_append(x_108, x_107); lean_dec(x_107); x_10 = x_98; -x_11 = x_99; -x_12 = lean_box(0); +x_11 = lean_box(0); +x_12 = x_102; x_13 = x_109; goto block_19; } @@ -1883,13 +1883,13 @@ if (lean_obj_tag(x_106) == 0) { lean_object* x_110; lean_dec_ref(x_101); -lean_dec(x_100); +lean_dec(x_97); x_110 = lean_ctor_get(x_106, 0); lean_inc(x_110); lean_dec_ref(x_106); x_10 = x_98; -x_11 = x_99; -x_12 = lean_box(0); +x_11 = lean_box(0); +x_12 = x_102; x_13 = x_110; goto block_19; } @@ -1899,11 +1899,11 @@ lean_object* x_111; x_111 = lean_ctor_get(x_106, 0); lean_inc(x_111); lean_dec_ref(x_106); -x_36 = x_98; -x_37 = x_99; -x_38 = x_100; +x_36 = x_97; +x_37 = x_98; +x_38 = lean_box(0); x_39 = x_101; -x_40 = lean_box(0); +x_40 = x_102; x_41 = x_111; goto block_96; } @@ -1951,9 +1951,9 @@ lean_dec(x_125); x_129 = lean_ctor_get(x_128, 0); lean_inc(x_129); lean_dec_ref(x_128); -x_26 = x_126; -x_27 = x_124; -x_28 = lean_box(0); +x_26 = x_124; +x_27 = lean_box(0); +x_28 = x_126; x_29 = x_129; goto block_35; } @@ -1971,9 +1971,9 @@ lean_dec(x_125); x_132 = lean_ctor_get(x_131, 0); lean_inc(x_132); lean_dec_ref(x_131); -x_26 = x_126; -x_27 = x_124; -x_28 = lean_box(0); +x_26 = x_124; +x_27 = lean_box(0); +x_28 = x_126; x_29 = x_132; goto block_35; } @@ -1989,9 +1989,9 @@ if (lean_obj_tag(x_135) == 0) { lean_dec(x_133); lean_dec(x_125); -x_20 = x_126; -x_21 = x_124; -x_22 = lean_box(0); +x_20 = x_124; +x_21 = lean_box(0); +x_22 = x_126; goto block_25; } else @@ -2004,12 +2004,12 @@ x_137 = l_Option_fromJson_x3f___at___00Lake_getUrl_x3f_spec__0(x_136); if (lean_obj_tag(x_137) == 0) { lean_dec_ref(x_137); -x_97 = x_133; -x_98 = x_126; -x_99 = x_124; -x_100 = x_118; +x_97 = x_118; +x_98 = x_124; +x_99 = lean_box(0); +x_100 = x_133; x_101 = x_125; -x_102 = lean_box(0); +x_102 = x_126; goto block_112; } else @@ -2017,12 +2017,12 @@ else if (lean_obj_tag(x_137) == 0) { lean_dec_ref(x_137); -x_97 = x_133; -x_98 = x_126; -x_99 = x_124; -x_100 = x_118; +x_97 = x_118; +x_98 = x_124; +x_99 = lean_box(0); +x_100 = x_133; x_101 = x_125; -x_102 = lean_box(0); +x_102 = x_126; goto block_112; } else @@ -2032,11 +2032,11 @@ lean_dec(x_133); x_138 = lean_ctor_get(x_137, 0); lean_inc(x_138); lean_dec_ref(x_137); -x_36 = x_126; +x_36 = x_118; x_37 = x_124; -x_38 = x_118; +x_38 = lean_box(0); x_39 = x_125; -x_40 = lean_box(0); +x_40 = x_126; x_41 = x_138; goto block_96; } diff --git a/stage0/stdlib/Lake/Util/Version.c b/stage0/stdlib/Lake/Util/Version.c index 0be979ad8897..1c471e92e7df 100644 --- a/stage0/stdlib/Lake/Util/Version.c +++ b/stage0/stdlib/Lake/Util/Version.c @@ -4552,7 +4552,7 @@ return x_2; LEAN_EXPORT lean_object* l_Lake_ToolchainVer_ofString(lean_object* x_1) { _start: { -lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_51; lean_object* x_52; lean_object* x_77; uint32_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_51; lean_object* x_52; lean_object* x_77; uint32_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; x_86 = 58; x_87 = lean_unsigned_to_nat(0u); x_88 = lean_string_utf8_byte_size(x_1); @@ -4581,12 +4581,12 @@ goto block_85; block_50: { lean_object* x_6; -lean_inc_ref(x_4); -x_6 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__0___redArg(x_4); +lean_inc_ref(x_2); +x_6 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__0___redArg(x_2); if (lean_obj_tag(x_6) == 1) { lean_object* x_7; lean_object* x_8; lean_object* x_9; -lean_dec_ref(x_4); +lean_dec_ref(x_2); x_7 = lean_ctor_get(x_6, 0); lean_inc(x_7); lean_dec_ref(x_6); @@ -4595,13 +4595,13 @@ lean_dec(x_7); x_9 = l_Lake_Date_ofString_x3f(x_8); if (lean_obj_tag(x_9) == 1) { -if (x_3 == 0) +if (x_4 == 0) { lean_object* x_10; lean_object* x_11; x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); lean_dec_ref(x_9); -x_11 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__1___redArg(x_2); +x_11 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__1___redArg(x_3); if (lean_obj_tag(x_11) == 1) { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; @@ -4670,7 +4670,7 @@ else { lean_object* x_25; lean_object* x_26; lean_dec(x_5); -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_dec_ref(x_1); x_25 = lean_ctor_get(x_9, 0); lean_inc(x_25); @@ -4684,7 +4684,7 @@ else lean_object* x_27; lean_dec(x_9); lean_dec(x_5); -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_inc_ref(x_1); x_27 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_27, 0, x_1); @@ -4696,7 +4696,7 @@ else { lean_object* x_28; lean_dec(x_6); -x_28 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__2___redArg(x_4); +x_28 = l_String_dropPrefix_x3f___at___00Lake_ToolchainVer_ofString_spec__2___redArg(x_2); if (lean_obj_tag(x_28) == 1) { lean_object* x_29; lean_object* x_30; @@ -4708,15 +4708,15 @@ x_30 = l_String_Slice_toNat_x3f(x_29); lean_dec(x_29); if (lean_obj_tag(x_30) == 1) { -if (x_3 == 0) +if (x_4 == 0) { lean_object* x_31; lean_object* x_32; uint8_t x_33; x_31 = lean_ctor_get(x_30, 0); lean_inc(x_31); lean_dec_ref(x_30); x_32 = l_Lake_ToolchainVer_prOrigin___closed__0; -x_33 = lean_string_dec_eq(x_2, x_32); -lean_dec_ref(x_2); +x_33 = lean_string_dec_eq(x_3, x_32); +lean_dec_ref(x_3); if (x_33 == 0) { lean_object* x_34; @@ -4738,7 +4738,7 @@ return x_35; else { lean_object* x_36; lean_object* x_37; -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_dec_ref(x_1); x_36 = lean_ctor_get(x_30, 0); lean_inc(x_36); @@ -4751,7 +4751,7 @@ else { lean_object* x_38; lean_dec(x_30); -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_inc_ref(x_1); x_38 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_38, 0, x_1); @@ -4769,15 +4769,15 @@ lean_inc_ref(x_1); x_41 = l___private_Lake_Util_Version_0__Lake_runVerParse___redArg(x_1, x_39, x_5, x_40); if (lean_obj_tag(x_41) == 1) { -if (x_3 == 0) +if (x_4 == 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); lean_dec_ref(x_41); x_43 = l_Lake_ToolchainVer_defaultOrigin___closed__0; -x_44 = lean_string_dec_eq(x_2, x_43); -lean_dec_ref(x_2); +x_44 = lean_string_dec_eq(x_3, x_43); +lean_dec_ref(x_3); if (x_44 == 0) { lean_object* x_45; @@ -4799,7 +4799,7 @@ return x_46; else { lean_object* x_47; lean_object* x_48; -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_dec_ref(x_1); x_47 = lean_ctor_get(x_41, 0); lean_inc(x_47); @@ -4812,7 +4812,7 @@ else { lean_object* x_49; lean_dec_ref(x_41); -lean_dec_ref(x_2); +lean_dec_ref(x_3); lean_inc_ref(x_1); x_49 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_49, 0, x_1); @@ -4834,9 +4834,9 @@ x_58 = l_Lake_ToolchainVer_ofString___closed__3; x_59 = lean_nat_dec_le(x_58, x_57); if (x_59 == 0) { -x_2 = x_51; -x_3 = x_55; -x_4 = x_52; +x_2 = x_52; +x_3 = x_51; +x_4 = x_55; x_5 = x_54; goto block_50; } @@ -4846,9 +4846,9 @@ uint8_t x_60; x_60 = lean_string_memcmp(x_52, x_56, x_54, x_54, x_58); if (x_60 == 0) { -x_2 = x_51; -x_3 = x_55; -x_4 = x_52; +x_2 = x_52; +x_3 = x_51; +x_4 = x_55; x_5 = x_54; goto block_50; } @@ -7108,7 +7108,7 @@ return x_5; LEAN_EXPORT uint8_t l_Lake_VerComparator_test(lean_object* x_1, lean_object* x_2) { _start: { -uint8_t x_3; lean_object* x_4; uint8_t x_5; uint8_t x_6; uint8_t x_7; lean_object* x_8; uint8_t x_9; lean_object* x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; lean_object* x_24; uint8_t x_25; uint8_t x_26; lean_object* x_27; uint8_t x_28; lean_object* x_33; uint8_t x_34; lean_object* x_35; uint8_t x_36; lean_object* x_41; uint8_t x_42; uint8_t x_43; lean_object* x_44; +uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; uint8_t x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; uint8_t x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_41; uint8_t x_42; uint8_t x_43; lean_object* x_44; x_41 = lean_ctor_get(x_1, 0); x_42 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); x_43 = lean_ctor_get_uint8(x_1, sizeof(void*)*1 + 1); @@ -7201,8 +7201,8 @@ goto block_48; block_13: { uint8_t x_10; -x_10 = l_Lake_instDecidableEqStdVer_decEq(x_8, x_4); -switch (x_7) { +x_10 = l_Lake_instDecidableEqStdVer_decEq(x_8, x_7); +switch (x_4) { case 0: { return x_5; @@ -7243,7 +7243,7 @@ return x_12; block_23: { uint8_t x_20; -x_20 = l_Lake_StdVer_compare(x_14, x_18); +x_20 = l_Lake_StdVer_compare(x_17, x_18); if (x_20 == 2) { uint8_t x_21; @@ -7274,7 +7274,7 @@ goto block_13; block_32: { uint8_t x_29; -x_29 = l_Lake_StdVer_compare(x_24, x_27); +x_29 = l_Lake_StdVer_compare(x_26, x_27); if (x_29 == 0) { uint8_t x_30; @@ -7303,7 +7303,7 @@ goto block_23; block_40: { uint8_t x_37; -x_37 = l_Lake_StdVer_compare(x_35, x_33); +x_37 = l_Lake_StdVer_compare(x_35, x_34); if (x_37 == 2) { uint8_t x_38; @@ -7335,8 +7335,8 @@ if (x_45 == 0) { uint8_t x_46; x_46 = 1; -x_33 = x_41; -x_34 = x_42; +x_33 = x_42; +x_34 = x_41; x_35 = x_44; x_36 = x_46; goto block_40; @@ -7345,8 +7345,8 @@ else { uint8_t x_47; x_47 = 0; -x_33 = x_41; -x_34 = x_42; +x_33 = x_42; +x_34 = x_41; x_35 = x_44; x_36 = x_47; goto block_40; @@ -11061,7 +11061,7 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lake_Util_Version_0__Lake_VerRange_parseM_parseWild(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_8; lean_object* x_13; 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_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_128; lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_149; uint8_t x_150; lean_object* x_151; lean_object* x_152; uint8_t x_167; lean_object* x_178; lean_object* x_179; lean_object* x_180; +lean_object* x_4; lean_object* x_8; lean_object* x_13; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; lean_object* x_134; lean_object* x_149; lean_object* x_150; uint8_t x_151; lean_object* x_152; uint8_t x_167; lean_object* x_178; lean_object* x_179; lean_object* x_180; x_17 = lean_unsigned_to_nat(0u); x_115 = l___private_Lake_Util_Version_0__Lake_parseVerComponents___closed__0; lean_inc(x_3); @@ -11152,15 +11152,15 @@ return x_15; block_114: { lean_object* x_25; -x_25 = l___private_Lake_Util_Version_0__Lake_parseVerComponent___redArg(x_23, x_24, x_22); +x_25 = l___private_Lake_Util_Version_0__Lake_parseVerComponent___redArg(x_22, x_24, x_18); lean_dec(x_24); -lean_dec_ref(x_23); +lean_dec_ref(x_22); if (lean_obj_tag(x_25) == 0) { -switch (lean_obj_tag(x_19)) { +switch (lean_obj_tag(x_21)) { case 2: { -switch (lean_obj_tag(x_18)) { +switch (lean_obj_tag(x_19)) { case 2: { lean_object* x_26; @@ -11175,19 +11175,19 @@ if (x_27 == 0) lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; x_28 = lean_ctor_get(x_25, 0); lean_dec(x_28); -x_29 = lean_ctor_get(x_19, 0); +x_29 = lean_ctor_get(x_21, 0); lean_inc(x_29); -lean_dec_ref(x_19); -x_30 = lean_ctor_get(x_18, 0); +lean_dec_ref(x_21); +x_30 = lean_ctor_get(x_19, 0); lean_inc(x_30); -lean_dec_ref(x_18); +lean_dec_ref(x_19); lean_inc(x_30); lean_inc(x_29); x_31 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); lean_ctor_set(x_31, 2, x_17); -x_32 = lean_nat_add(x_30, x_21); +x_32 = lean_nat_add(x_30, x_20); lean_dec(x_30); x_33 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_33, 0, x_29); @@ -11204,7 +11204,7 @@ x_37 = 3; x_38 = lean_alloc_ctor(0, 1, 2); lean_ctor_set(x_38, 0, x_35); lean_ctor_set_uint8(x_38, sizeof(void*)*1, x_37); -lean_ctor_set_uint8(x_38, sizeof(void*)*1 + 1, x_20); +lean_ctor_set_uint8(x_38, sizeof(void*)*1 + 1, x_23); x_39 = lean_array_push(x_2, x_38); x_40 = 0; x_41 = 1; @@ -11222,19 +11222,19 @@ lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean x_44 = lean_ctor_get(x_25, 1); lean_inc(x_44); lean_dec(x_25); -x_45 = lean_ctor_get(x_19, 0); +x_45 = lean_ctor_get(x_21, 0); lean_inc(x_45); -lean_dec_ref(x_19); -x_46 = lean_ctor_get(x_18, 0); +lean_dec_ref(x_21); +x_46 = lean_ctor_get(x_19, 0); lean_inc(x_46); -lean_dec_ref(x_18); +lean_dec_ref(x_19); lean_inc(x_46); lean_inc(x_45); x_47 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_46); lean_ctor_set(x_47, 2, x_17); -x_48 = lean_nat_add(x_46, x_21); +x_48 = lean_nat_add(x_46, x_20); lean_dec(x_46); x_49 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_49, 0, x_45); @@ -11251,7 +11251,7 @@ x_53 = 3; x_54 = lean_alloc_ctor(0, 1, 2); lean_ctor_set(x_54, 0, x_51); lean_ctor_set_uint8(x_54, sizeof(void*)*1, x_53); -lean_ctor_set_uint8(x_54, sizeof(void*)*1 + 1, x_20); +lean_ctor_set_uint8(x_54, sizeof(void*)*1 + 1, x_23); x_55 = lean_array_push(x_2, x_54); x_56 = 0; x_57 = 1; @@ -11270,8 +11270,8 @@ else { lean_object* x_61; lean_dec(x_26); +lean_dec_ref(x_21); lean_dec_ref(x_19); -lean_dec_ref(x_18); lean_dec_ref(x_2); x_61 = lean_ctor_get(x_25, 1); lean_inc(x_61); @@ -11289,7 +11289,7 @@ if (lean_obj_tag(x_62) == 2) { lean_object* x_63; lean_dec_ref(x_62); -lean_dec_ref(x_19); +lean_dec_ref(x_21); lean_dec_ref(x_2); x_63 = lean_ctor_get(x_25, 1); lean_inc(x_63); @@ -11307,15 +11307,15 @@ if (x_64 == 0) lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; x_65 = lean_ctor_get(x_25, 0); lean_dec(x_65); -x_66 = lean_ctor_get(x_19, 0); +x_66 = lean_ctor_get(x_21, 0); lean_inc(x_66); -lean_dec_ref(x_19); +lean_dec_ref(x_21); lean_inc(x_66); x_67 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_67, 0, x_66); lean_ctor_set(x_67, 1, x_17); lean_ctor_set(x_67, 2, x_17); -x_68 = lean_nat_add(x_66, x_21); +x_68 = lean_nat_add(x_66, x_20); lean_dec(x_66); x_69 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_69, 0, x_68); @@ -11332,7 +11332,7 @@ x_73 = 3; x_74 = lean_alloc_ctor(0, 1, 2); lean_ctor_set(x_74, 0, x_71); lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_73); -lean_ctor_set_uint8(x_74, sizeof(void*)*1 + 1, x_20); +lean_ctor_set_uint8(x_74, sizeof(void*)*1 + 1, x_23); x_75 = lean_array_push(x_2, x_74); x_76 = 0; x_77 = 1; @@ -11350,15 +11350,15 @@ lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean x_80 = lean_ctor_get(x_25, 1); lean_inc(x_80); lean_dec(x_25); -x_81 = lean_ctor_get(x_19, 0); +x_81 = lean_ctor_get(x_21, 0); lean_inc(x_81); -lean_dec_ref(x_19); +lean_dec_ref(x_21); lean_inc(x_81); x_82 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_82, 0, x_81); lean_ctor_set(x_82, 1, x_17); lean_ctor_set(x_82, 2, x_17); -x_83 = lean_nat_add(x_81, x_21); +x_83 = lean_nat_add(x_81, x_20); lean_dec(x_81); x_84 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_84, 0, x_83); @@ -11375,7 +11375,7 @@ x_88 = 3; x_89 = lean_alloc_ctor(0, 1, 2); lean_ctor_set(x_89, 0, x_86); lean_ctor_set_uint8(x_89, sizeof(void*)*1, x_88); -lean_ctor_set_uint8(x_89, sizeof(void*)*1 + 1, x_20); +lean_ctor_set_uint8(x_89, sizeof(void*)*1 + 1, x_23); x_90 = lean_array_push(x_2, x_89); x_91 = 0; x_92 = 1; @@ -11394,8 +11394,8 @@ return x_95; default: { lean_object* x_96; -lean_dec_ref(x_19); -lean_dec(x_18); +lean_dec_ref(x_21); +lean_dec(x_19); lean_dec_ref(x_2); x_96 = lean_ctor_get(x_25, 1); lean_inc(x_96); @@ -11414,7 +11414,7 @@ if (lean_obj_tag(x_97) == 2) { lean_object* x_98; lean_dec_ref(x_97); -lean_dec(x_18); +lean_dec(x_19); lean_dec_ref(x_2); x_98 = lean_ctor_get(x_25, 1); lean_inc(x_98); @@ -11425,10 +11425,10 @@ goto block_16; else { lean_dec(x_97); -if (lean_obj_tag(x_18) == 2) +if (lean_obj_tag(x_19) == 2) { uint8_t x_99; -lean_dec_ref(x_18); +lean_dec_ref(x_19); lean_dec_ref(x_2); x_99 = !lean_is_exclusive(x_25); if (x_99 == 0) @@ -11457,7 +11457,7 @@ return x_104; else { lean_object* x_105; -lean_dec(x_18); +lean_dec(x_19); x_105 = lean_ctor_get(x_25, 1); lean_inc(x_105); lean_dec_ref(x_25); @@ -11468,8 +11468,8 @@ goto block_12; } default: { -lean_dec(x_19); -if (lean_obj_tag(x_18) == 1) +lean_dec(x_21); +if (lean_obj_tag(x_19) == 1) { lean_object* x_106; x_106 = lean_ctor_get(x_25, 0); @@ -11499,7 +11499,7 @@ goto block_12; else { lean_object* x_109; -lean_dec(x_18); +lean_dec(x_19); x_109 = lean_ctor_get(x_25, 1); lean_inc(x_109); lean_dec_ref(x_25); @@ -11512,8 +11512,8 @@ goto block_12; else { uint8_t x_110; +lean_dec(x_21); lean_dec(x_19); -lean_dec(x_18); lean_dec_ref(x_2); x_110 = !lean_is_exclusive(x_25); if (x_110 == 0) @@ -11557,9 +11557,9 @@ return x_126; block_148: { lean_object* x_135; -x_135 = l___private_Lake_Util_Version_0__Lake_parseVerComponent___redArg(x_129, x_134, x_133); +x_135 = l___private_Lake_Util_Version_0__Lake_parseVerComponent___redArg(x_130, x_134, x_128); lean_dec(x_134); -lean_dec_ref(x_129); +lean_dec_ref(x_130); if (lean_obj_tag(x_135) == 0) { lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; uint8_t x_140; @@ -11570,19 +11570,19 @@ lean_inc(x_137); lean_dec_ref(x_135); x_138 = l_Lake_instReprSemVerCore_repr___redArg___closed__12; x_139 = lean_unsigned_to_nat(2u); -x_140 = lean_nat_dec_lt(x_139, x_132); -lean_dec(x_132); +x_140 = lean_nat_dec_lt(x_139, x_129); +lean_dec(x_129); if (x_140 == 0) { lean_object* x_141; lean_dec(x_117); x_141 = lean_box(0); -x_18 = x_136; -x_19 = x_128; -x_20 = x_131; -x_21 = x_130; -x_22 = x_137; -x_23 = x_138; +x_18 = x_137; +x_19 = x_136; +x_20 = x_132; +x_21 = x_131; +x_22 = x_138; +x_23 = x_133; x_24 = x_141; goto block_114; } @@ -11593,12 +11593,12 @@ x_142 = lean_array_fget(x_117, x_139); lean_dec(x_117); x_143 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_143, 0, x_142); -x_18 = x_136; -x_19 = x_128; -x_20 = x_131; -x_21 = x_130; -x_22 = x_137; -x_23 = x_138; +x_18 = x_137; +x_19 = x_136; +x_20 = x_132; +x_21 = x_131; +x_22 = x_138; +x_23 = x_133; x_24 = x_143; goto block_114; } @@ -11606,8 +11606,8 @@ goto block_114; else { uint8_t x_144; -lean_dec(x_132); -lean_dec(x_128); +lean_dec(x_131); +lean_dec(x_129); lean_dec(x_117); lean_dec_ref(x_2); x_144 = !lean_is_exclusive(x_135); @@ -11646,17 +11646,17 @@ lean_inc(x_155); lean_dec_ref(x_153); x_156 = l_Lake_instReprSemVerCore_repr___redArg___closed__10; x_157 = lean_unsigned_to_nat(1u); -x_158 = lean_nat_dec_lt(x_157, x_151); +x_158 = lean_nat_dec_lt(x_157, x_150); if (x_158 == 0) { lean_object* x_159; x_159 = lean_box(0); -x_128 = x_154; -x_129 = x_156; -x_130 = x_157; -x_131 = x_150; -x_132 = x_151; -x_133 = x_155; +x_128 = x_155; +x_129 = x_150; +x_130 = x_156; +x_131 = x_154; +x_132 = x_157; +x_133 = x_151; x_134 = x_159; goto block_148; } @@ -11667,12 +11667,12 @@ x_160 = lean_array_fget_borrowed(x_117, x_157); lean_inc(x_160); x_161 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_161, 0, x_160); -x_128 = x_154; -x_129 = x_156; -x_130 = x_157; -x_131 = x_150; -x_132 = x_151; -x_133 = x_155; +x_128 = x_155; +x_129 = x_150; +x_130 = x_156; +x_131 = x_154; +x_132 = x_157; +x_133 = x_151; x_134 = x_161; goto block_148; } @@ -11680,7 +11680,7 @@ goto block_148; else { uint8_t x_162; -lean_dec(x_151); +lean_dec(x_150); lean_dec(x_117); lean_dec_ref(x_2); x_162 = !lean_is_exclusive(x_153); @@ -11724,8 +11724,8 @@ if (x_173 == 0) lean_object* x_174; x_174 = lean_box(0); x_149 = x_172; -x_150 = x_167; -x_151 = x_168; +x_150 = x_168; +x_151 = x_167; x_152 = x_174; goto block_166; } @@ -11737,8 +11737,8 @@ lean_inc(x_175); x_176 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_176, 0, x_175); x_149 = x_172; -x_150 = x_167; -x_151 = x_168; +x_150 = x_168; +x_151 = x_167; x_152 = x_176; goto block_166; } diff --git a/stage0/stdlib/Lean.c b/stage0/stdlib/Lean.c index a75c38f6ebe0..1ad710200b7a 100644 --- a/stage0/stdlib/Lean.c +++ b/stage0/stdlib/Lean.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean -// Imports: public import Init public import Lean.Data public import Lean.Compiler public import Lean.Environment public import Lean.Modifiers public import Lean.ProjFns public import Lean.Runtime public import Lean.ResolveName public import Lean.Attributes public import Lean.Parser public import Lean.ReducibilityAttrs public import Lean.Elab public import Lean.Class public import Lean.LocalContext public import Lean.MetavarContext public import Lean.AuxRecursor public import Lean.Meta public import Lean.Util public import Lean.Structure public import Lean.PrettyPrinter public import Lean.CoreM public import Lean.ReservedNameAction public import Lean.InternalExceptionId public import Lean.Server public import Lean.ScopedEnvExtension public import Lean.DocString public import Lean.DeclarationRange public import Lean.LoadDynlib public import Lean.Widget public import Lean.Log public import Lean.Linter public import Lean.SubExpr public import Lean.LabelAttribute public import Lean.AddDecl public import Lean.Replay public import Lean.PrivateName public import Lean.LibrarySuggestions public import Lean.Namespace public import Lean.EnvExtension public import Lean.ErrorExplanation public import Lean.ErrorExplanations public import Lean.DefEqAttrib public import Lean.Shell public import Lean.ExtraModUses +// Imports: public import Init public import Lean.Data public import Lean.Compiler public import Lean.Environment public import Lean.Modifiers public import Lean.ProjFns public import Lean.Runtime public import Lean.ResolveName public import Lean.Attributes public import Lean.Parser public import Lean.ReducibilityAttrs public import Lean.Elab public import Lean.Class public import Lean.LocalContext public import Lean.MetavarContext public import Lean.AuxRecursor public import Lean.Meta public import Lean.Util public import Lean.Structure public import Lean.PrettyPrinter public import Lean.CoreM public import Lean.ReservedNameAction public import Lean.InternalExceptionId public import Lean.Server public import Lean.ScopedEnvExtension public import Lean.DocString public import Lean.DeclarationRange public import Lean.LoadDynlib public import Lean.Widget public import Lean.Log public import Lean.Linter public import Lean.SubExpr public import Lean.LabelAttribute public import Lean.AddDecl public import Lean.Replay public import Lean.PrivateName public import Lean.LibrarySuggestions public import Lean.Namespace public import Lean.EnvExtension public import Lean.ErrorExplanation public import Lean.ErrorExplanations public import Lean.DefEqAttrib public import Lean.Shell public import Lean.ExtraModUses public import Lean.AllowNativeDecide #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -57,6 +57,7 @@ lean_object* initialize_Lean_ErrorExplanations(uint8_t builtin); lean_object* initialize_Lean_DefEqAttrib(uint8_t builtin); lean_object* initialize_Lean_Shell(uint8_t builtin); lean_object* initialize_Lean_ExtraModUses(uint8_t builtin); +lean_object* initialize_Lean_AllowNativeDecide(uint8_t builtin); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean(uint8_t builtin) { lean_object * res; @@ -194,6 +195,9 @@ lean_dec_ref(res); res = initialize_Lean_ExtraModUses(builtin); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_AllowNativeDecide(builtin); +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/Lean/AllowNativeDecide.c b/stage0/stdlib/Lean/AllowNativeDecide.c new file mode 100644 index 000000000000..1164ee135cce --- /dev/null +++ b/stage0/stdlib/Lean/AllowNativeDecide.c @@ -0,0 +1,154 @@ +// Lean compiler output +// Module: Lean.AllowNativeDecide +// Imports: public import Lean.Attributes +#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_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +static lean_object* l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +LEAN_EXPORT lean_object* l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2____boxed(lean_object*); +static lean_object* l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +LEAN_EXPORT lean_object* l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_object* l_Lean_registerTagAttribute(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); +static lean_object* l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +LEAN_EXPORT lean_object* l___private_Lean_AllowNativeDecide_0__Lean_allowNativeDecideAttr; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +lean_object* l_Lean_Name_mkStr1(lean_object*); +static lean_object* l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +LEAN_EXPORT lean_object* l_Lean_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2____boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_box(0); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("allow_native_decide", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_2 = l_Lean_Name_mkStr1(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mark definition as allowed to be used in `native_decide` computations", 69, 69); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("allowNativeDecideAttr", 21, 21); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_2 = l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_3 = l_Lean_Name_mkStr2(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_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_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec_ref(x_2); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_() { +_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; lean_object* x_8; +x_2 = lean_alloc_closure((void*)(l_Lean_initFn___lam__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2____boxed), 4, 0); +x_3 = l_Lean_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_4 = l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_5 = l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_; +x_6 = 0; +x_7 = lean_box(2); +x_8 = l_Lean_registerTagAttribute(x_3, x_4, x_2, x_5, x_6, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2____boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +return x_2; +} +} +lean_object* initialize_Lean_Attributes(uint8_t builtin); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_AllowNativeDecide(uint8_t builtin) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Attributes(builtin); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__0_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +l_Lean_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__1_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__2_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__3_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__4_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_ = _init_l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +lean_mark_persistent(l_Lean_initFn___closed__5_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_); +if (builtin) {res = l_Lean_initFn_00___x40_Lean_AllowNativeDecide_3406689909____hygCtx___hyg_2_(); +if (lean_io_result_is_error(res)) return res; +l___private_Lean_AllowNativeDecide_0__Lean_allowNativeDecideAttr = lean_io_result_get_value(res); +lean_mark_persistent(l___private_Lean_AllowNativeDecide_0__Lean_allowNativeDecideAttr); +lean_dec_ref(res); +}return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Basic.c b/stage0/stdlib/Lean/Compiler/LCNF/Basic.c index 9419d3de238a..11c5b3fb195c 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Basic.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Basic.c @@ -7999,8 +7999,8 @@ if (x_6 == 0) lean_object* x_7; lean_dec_ref(x_3); x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_4); -lean_ctor_set(x_7, 1, x_5); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_4); return x_7; } else @@ -8017,8 +8017,8 @@ if (x_11 == 0) lean_object* x_12; lean_dec_ref(x_3); x_12 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_12, 0, x_9); -lean_ctor_set(x_12, 1, x_10); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_9); return x_12; } else @@ -8046,8 +8046,8 @@ x_21 = lean_ptr_addr(x_17); x_22 = lean_usize_dec_eq(x_20, x_21); if (x_22 == 0) { -x_4 = x_16; -x_5 = x_17; +x_4 = x_17; +x_5 = x_16; x_6 = x_22; goto block_8; } @@ -8057,8 +8057,8 @@ size_t x_23; size_t x_24; uint8_t x_25; x_23 = lean_ptr_addr(x_18); x_24 = lean_ptr_addr(x_16); x_25 = lean_usize_dec_eq(x_23, x_24); -x_4 = x_16; -x_5 = x_17; +x_4 = x_17; +x_5 = x_16; x_6 = x_25; goto block_8; } @@ -8073,8 +8073,8 @@ x_29 = lean_ptr_addr(x_17); x_30 = lean_usize_dec_eq(x_28, x_29); if (x_30 == 0) { -x_9 = x_16; -x_10 = x_17; +x_9 = x_17; +x_10 = x_16; x_11 = x_30; goto block_13; } @@ -8084,8 +8084,8 @@ size_t x_31; size_t x_32; uint8_t x_33; x_31 = lean_ptr_addr(x_26); x_32 = lean_ptr_addr(x_16); x_33 = lean_usize_dec_eq(x_31, x_32); -x_9 = x_16; -x_10 = x_17; +x_9 = x_17; +x_10 = x_16; x_11 = x_33; goto block_13; } diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c b/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c index be9ad2015d8f..5fc390f3260f 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c @@ -16123,27 +16123,27 @@ goto block_219; block_173: { uint8_t x_83; -x_83 = l_Lean_Expr_hasLooseBVars(x_72); +x_83 = l_Lean_Expr_hasLooseBVars(x_73); if (x_83 == 0) { uint8_t x_84; -x_84 = l_Lean_Expr_hasFVar(x_72); +x_84 = l_Lean_Expr_hasFVar(x_73); if (x_84 == 0) { lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; size_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_85 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_72, x_81); +x_85 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_73, x_81); x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); lean_dec_ref(x_85); x_87 = lean_box(0); -lean_inc(x_73); -x_88 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_73, x_87); -x_89 = lean_array_size(x_70); +lean_inc(x_72); +x_88 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_72, x_87); +x_89 = lean_array_size(x_74); x_90 = 0; -lean_inc_ref(x_70); -x_91 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_89, x_90, x_70); -x_92 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_74, x_50); -lean_dec_ref(x_74); +lean_inc_ref(x_74); +x_91 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_89, x_90, x_74); +x_92 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_75, x_50); +lean_dec_ref(x_75); x_93 = l_Array_append___redArg(x_91, x_92); lean_dec_ref(x_92); if (lean_obj_tag(x_86) == 1) @@ -16152,9 +16152,9 @@ lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint lean_dec_ref(x_78); lean_dec(x_77); lean_dec_ref(x_76); -lean_dec_ref(x_75); -lean_dec(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_74); +lean_dec_ref(x_73); +lean_dec(x_72); lean_dec_ref(x_71); lean_dec_ref(x_70); lean_dec(x_68); @@ -16176,9 +16176,9 @@ if (x_98 == 0) lean_dec(x_81); lean_dec_ref(x_80); lean_dec(x_79); -x_9 = x_93; -x_10 = x_94; -x_11 = x_88; +x_9 = x_88; +x_10 = x_93; +x_11 = x_94; x_12 = lean_box(0); goto block_16; } @@ -16196,9 +16196,9 @@ lean_dec(x_81); lean_dec_ref(x_80); lean_dec(x_79); lean_dec_ref(x_102); -x_9 = x_93; -x_10 = x_94; -x_11 = x_88; +x_9 = x_88; +x_10 = x_93; +x_11 = x_94; x_12 = lean_box(0); goto block_16; } @@ -16211,7 +16211,7 @@ lean_inc(x_81); lean_inc_ref(x_80); lean_inc(x_79); lean_inc_ref(x_78); -x_103 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_68, x_49, x_75, x_70, x_71, x_73, x_76, x_77, x_78, x_79, x_80, x_81); +x_103 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_68, x_49, x_71, x_74, x_70, x_72, x_76, x_77, x_78, x_79, x_80, x_81); if (lean_obj_tag(x_103) == 0) { lean_object* x_104; size_t x_105; uint8_t x_106; uint8_t x_107; lean_object* x_108; @@ -16231,7 +16231,7 @@ lean_inc(x_109); lean_dec_ref(x_108); x_110 = lean_ctor_get(x_104, 0); lean_inc(x_110); -x_111 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_72, x_110, x_81); +x_111 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_73, x_110, x_81); lean_dec_ref(x_111); lean_inc(x_104); x_112 = l_Lean_Compiler_LCNF_Decl_saveBase___redArg(x_104, x_81); @@ -16311,10 +16311,10 @@ lean_dec(x_81); lean_dec_ref(x_80); lean_dec(x_79); lean_dec_ref(x_78); -x_17 = x_93; -x_18 = x_129; -x_19 = x_109; -x_20 = x_88; +x_17 = x_88; +x_18 = x_93; +x_19 = x_129; +x_20 = x_109; x_21 = x_77; x_22 = lean_box(0); goto block_47; @@ -16353,10 +16353,10 @@ lean_dec(x_81); lean_dec_ref(x_80); lean_dec(x_79); lean_dec_ref(x_144); -x_17 = x_93; -x_18 = x_129; -x_19 = x_109; -x_20 = x_88; +x_17 = x_88; +x_18 = x_93; +x_19 = x_129; +x_20 = x_109; x_21 = x_77; x_22 = lean_box(0); goto block_47; @@ -16550,7 +16550,7 @@ lean_dec_ref(x_80); lean_dec(x_79); lean_dec_ref(x_78); lean_dec(x_77); -lean_dec_ref(x_72); +lean_dec_ref(x_73); lean_dec(x_62); lean_dec(x_54); x_163 = !lean_is_exclusive(x_108); @@ -16580,7 +16580,7 @@ lean_dec_ref(x_80); lean_dec(x_79); lean_dec_ref(x_78); lean_dec(x_77); -lean_dec_ref(x_72); +lean_dec_ref(x_73); lean_dec(x_62); lean_dec(x_54); x_166 = !lean_is_exclusive(x_103); @@ -16606,8 +16606,8 @@ else lean_object* x_169; lean_object* x_170; lean_dec_ref(x_75); lean_dec_ref(x_74); -lean_dec(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_73); +lean_dec(x_72); lean_dec_ref(x_71); lean_dec_ref(x_70); lean_dec(x_68); @@ -16625,8 +16625,8 @@ else lean_object* x_171; lean_object* x_172; lean_dec_ref(x_75); lean_dec_ref(x_74); -lean_dec(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_73); +lean_dec(x_72); lean_dec_ref(x_71); lean_dec_ref(x_70); lean_dec(x_68); @@ -16702,12 +16702,12 @@ lean_dec(x_199); if (x_200 == 0) { lean_free_object(x_194); -x_70 = x_187; -x_71 = x_188; -x_72 = x_196; -x_73 = x_197; -x_74 = x_182; -x_75 = x_186; +x_70 = x_188; +x_71 = x_186; +x_72 = x_197; +x_73 = x_196; +x_74 = x_187; +x_75 = x_182; x_76 = x_175; x_77 = x_176; x_78 = x_177; @@ -16728,12 +16728,12 @@ lean_ctor_set(x_194, 1, x_202); lean_ctor_set(x_194, 0, x_201); x_203 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_174, x_194, x_178, x_179, x_180); lean_dec_ref(x_203); -x_70 = x_187; -x_71 = x_188; -x_72 = x_196; -x_73 = x_197; -x_74 = x_182; -x_75 = x_186; +x_70 = x_188; +x_71 = x_186; +x_72 = x_197; +x_73 = x_196; +x_74 = x_187; +x_75 = x_182; x_76 = x_175; x_77 = x_176; x_78 = x_177; @@ -16760,12 +16760,12 @@ x_208 = lean_unbox(x_207); lean_dec(x_207); if (x_208 == 0) { -x_70 = x_187; -x_71 = x_188; -x_72 = x_204; -x_73 = x_205; -x_74 = x_182; -x_75 = x_186; +x_70 = x_188; +x_71 = x_186; +x_72 = x_205; +x_73 = x_204; +x_74 = x_187; +x_75 = x_182; x_76 = x_175; x_77 = x_176; x_78 = x_177; @@ -16786,12 +16786,12 @@ lean_ctor_set(x_211, 0, x_209); lean_ctor_set(x_211, 1, x_210); x_212 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_174, x_211, x_178, x_179, x_180); lean_dec_ref(x_212); -x_70 = x_187; -x_71 = x_188; -x_72 = x_204; -x_73 = x_205; -x_74 = x_182; -x_75 = x_186; +x_70 = x_188; +x_71 = x_186; +x_72 = x_205; +x_73 = x_204; +x_74 = x_187; +x_75 = x_182; x_76 = x_175; x_77 = x_176; x_78 = x_177; @@ -17034,27 +17034,27 @@ goto block_396; block_358: { uint8_t x_268; -x_268 = l_Lean_Expr_hasLooseBVars(x_257); +x_268 = l_Lean_Expr_hasLooseBVars(x_258); if (x_268 == 0) { uint8_t x_269; -x_269 = l_Lean_Expr_hasFVar(x_257); +x_269 = l_Lean_Expr_hasFVar(x_258); if (x_269 == 0) { lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; size_t x_274; size_t x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; -x_270 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_257, x_266); +x_270 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_258, x_266); x_271 = lean_ctor_get(x_270, 0); lean_inc(x_271); lean_dec_ref(x_270); x_272 = lean_box(0); -lean_inc(x_258); -x_273 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_258, x_272); -x_274 = lean_array_size(x_255); +lean_inc(x_257); +x_273 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_257, x_272); +x_274 = lean_array_size(x_259); x_275 = 0; -lean_inc_ref(x_255); -x_276 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_274, x_275, x_255); -x_277 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_259, x_50); -lean_dec_ref(x_259); +lean_inc_ref(x_259); +x_276 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_274, x_275, x_259); +x_277 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_260, x_50); +lean_dec_ref(x_260); x_278 = l_Array_append___redArg(x_276, x_277); lean_dec_ref(x_277); if (lean_obj_tag(x_271) == 1) @@ -17063,9 +17063,9 @@ lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_dec_ref(x_263); lean_dec(x_262); lean_dec_ref(x_261); -lean_dec_ref(x_260); -lean_dec(x_258); -lean_dec_ref(x_257); +lean_dec_ref(x_259); +lean_dec_ref(x_258); +lean_dec(x_257); lean_dec_ref(x_256); lean_dec_ref(x_255); lean_dec(x_253); @@ -17087,9 +17087,9 @@ if (x_283 == 0) lean_dec(x_266); lean_dec_ref(x_265); lean_dec(x_264); -x_9 = x_278; -x_10 = x_279; -x_11 = x_273; +x_9 = x_273; +x_10 = x_278; +x_11 = x_279; x_12 = lean_box(0); goto block_16; } @@ -17107,9 +17107,9 @@ lean_dec(x_266); lean_dec_ref(x_265); lean_dec(x_264); lean_dec_ref(x_287); -x_9 = x_278; -x_10 = x_279; -x_11 = x_273; +x_9 = x_273; +x_10 = x_278; +x_11 = x_279; x_12 = lean_box(0); goto block_16; } @@ -17122,7 +17122,7 @@ lean_inc(x_266); lean_inc_ref(x_265); lean_inc(x_264); lean_inc_ref(x_263); -x_288 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_253, x_49, x_260, x_255, x_256, x_258, x_261, x_262, x_263, x_264, x_265, x_266); +x_288 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_253, x_49, x_256, x_259, x_255, x_257, x_261, x_262, x_263, x_264, x_265, x_266); if (lean_obj_tag(x_288) == 0) { lean_object* x_289; size_t x_290; uint8_t x_291; uint8_t x_292; lean_object* x_293; @@ -17142,7 +17142,7 @@ lean_inc(x_294); lean_dec_ref(x_293); x_295 = lean_ctor_get(x_289, 0); lean_inc(x_295); -x_296 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_257, x_295, x_266); +x_296 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_258, x_295, x_266); lean_dec_ref(x_296); lean_inc(x_289); x_297 = l_Lean_Compiler_LCNF_Decl_saveBase___redArg(x_289, x_266); @@ -17222,10 +17222,10 @@ lean_dec(x_266); lean_dec_ref(x_265); lean_dec(x_264); lean_dec_ref(x_263); -x_17 = x_278; -x_18 = x_314; -x_19 = x_294; -x_20 = x_273; +x_17 = x_273; +x_18 = x_278; +x_19 = x_314; +x_20 = x_294; x_21 = x_262; x_22 = lean_box(0); goto block_47; @@ -17264,10 +17264,10 @@ lean_dec(x_266); lean_dec_ref(x_265); lean_dec(x_264); lean_dec_ref(x_329); -x_17 = x_278; -x_18 = x_314; -x_19 = x_294; -x_20 = x_273; +x_17 = x_273; +x_18 = x_278; +x_19 = x_314; +x_20 = x_294; x_21 = x_262; x_22 = lean_box(0); goto block_47; @@ -17467,7 +17467,7 @@ lean_dec_ref(x_265); lean_dec(x_264); lean_dec_ref(x_263); lean_dec(x_262); -lean_dec_ref(x_257); +lean_dec_ref(x_258); lean_dec(x_62); lean_dec(x_54); x_348 = lean_ctor_get(x_293, 0); @@ -17498,7 +17498,7 @@ lean_dec_ref(x_265); lean_dec(x_264); lean_dec_ref(x_263); lean_dec(x_262); -lean_dec_ref(x_257); +lean_dec_ref(x_258); lean_dec(x_62); lean_dec(x_54); x_351 = lean_ctor_get(x_288, 0); @@ -17525,8 +17525,8 @@ else lean_object* x_354; lean_object* x_355; lean_dec_ref(x_260); lean_dec_ref(x_259); -lean_dec(x_258); -lean_dec_ref(x_257); +lean_dec_ref(x_258); +lean_dec(x_257); lean_dec_ref(x_256); lean_dec_ref(x_255); lean_dec(x_253); @@ -17544,8 +17544,8 @@ else lean_object* x_356; lean_object* x_357; lean_dec_ref(x_260); lean_dec_ref(x_259); -lean_dec(x_258); -lean_dec_ref(x_257); +lean_dec_ref(x_258); +lean_dec(x_257); lean_dec_ref(x_256); lean_dec_ref(x_255); lean_dec(x_253); @@ -17627,12 +17627,12 @@ lean_dec(x_384); if (x_385 == 0) { lean_dec(x_382); -x_255 = x_372; -x_256 = x_373; -x_257 = x_380; -x_258 = x_381; -x_259 = x_367; -x_260 = x_371; +x_255 = x_373; +x_256 = x_371; +x_257 = x_381; +x_258 = x_380; +x_259 = x_372; +x_260 = x_367; x_261 = x_360; x_262 = x_361; x_263 = x_362; @@ -17658,12 +17658,12 @@ lean_ctor_set(x_388, 0, x_386); lean_ctor_set(x_388, 1, x_387); x_389 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_359, x_388, x_363, x_364, x_365); lean_dec_ref(x_389); -x_255 = x_372; -x_256 = x_373; -x_257 = x_380; -x_258 = x_381; -x_259 = x_367; -x_260 = x_371; +x_255 = x_373; +x_256 = x_371; +x_257 = x_381; +x_258 = x_380; +x_259 = x_372; +x_260 = x_367; x_261 = x_360; x_262 = x_361; x_263 = x_362; @@ -17984,27 +17984,27 @@ goto block_584; block_546: { uint8_t x_456; -x_456 = l_Lean_Expr_hasLooseBVars(x_445); +x_456 = l_Lean_Expr_hasLooseBVars(x_446); if (x_456 == 0) { uint8_t x_457; -x_457 = l_Lean_Expr_hasFVar(x_445); +x_457 = l_Lean_Expr_hasFVar(x_446); if (x_457 == 0) { lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; size_t x_462; size_t x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; -x_458 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_445, x_454); +x_458 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_446, x_454); x_459 = lean_ctor_get(x_458, 0); lean_inc(x_459); lean_dec_ref(x_458); x_460 = lean_box(0); -lean_inc(x_446); -x_461 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_446, x_460); -x_462 = lean_array_size(x_443); +lean_inc(x_445); +x_461 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_445, x_460); +x_462 = lean_array_size(x_447); x_463 = 0; -lean_inc_ref(x_443); -x_464 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_462, x_463, x_443); -x_465 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_447, x_50); -lean_dec_ref(x_447); +lean_inc_ref(x_447); +x_464 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_462, x_463, x_447); +x_465 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_448, x_50); +lean_dec_ref(x_448); x_466 = l_Array_append___redArg(x_464, x_465); lean_dec_ref(x_465); if (lean_obj_tag(x_459) == 1) @@ -18013,9 +18013,9 @@ lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_dec_ref(x_451); lean_dec(x_450); lean_dec_ref(x_449); -lean_dec_ref(x_448); -lean_dec(x_446); -lean_dec_ref(x_445); +lean_dec_ref(x_447); +lean_dec_ref(x_446); +lean_dec(x_445); lean_dec_ref(x_444); lean_dec_ref(x_443); lean_dec(x_441); @@ -18037,9 +18037,9 @@ if (x_471 == 0) lean_dec(x_454); lean_dec_ref(x_453); lean_dec(x_452); -x_9 = x_466; -x_10 = x_467; -x_11 = x_461; +x_9 = x_461; +x_10 = x_466; +x_11 = x_467; x_12 = lean_box(0); goto block_16; } @@ -18057,9 +18057,9 @@ lean_dec(x_454); lean_dec_ref(x_453); lean_dec(x_452); lean_dec_ref(x_475); -x_9 = x_466; -x_10 = x_467; -x_11 = x_461; +x_9 = x_461; +x_10 = x_466; +x_11 = x_467; x_12 = lean_box(0); goto block_16; } @@ -18072,7 +18072,7 @@ lean_inc(x_454); lean_inc_ref(x_453); lean_inc(x_452); lean_inc_ref(x_451); -x_476 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_441, x_49, x_448, x_443, x_444, x_446, x_449, x_450, x_451, x_452, x_453, x_454); +x_476 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_441, x_49, x_444, x_447, x_443, x_445, x_449, x_450, x_451, x_452, x_453, x_454); if (lean_obj_tag(x_476) == 0) { lean_object* x_477; size_t x_478; uint8_t x_479; uint8_t x_480; lean_object* x_481; @@ -18092,7 +18092,7 @@ lean_inc(x_482); lean_dec_ref(x_481); x_483 = lean_ctor_get(x_477, 0); lean_inc(x_483); -x_484 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_445, x_483, x_454); +x_484 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_446, x_483, x_454); lean_dec_ref(x_484); lean_inc(x_477); x_485 = l_Lean_Compiler_LCNF_Decl_saveBase___redArg(x_477, x_454); @@ -18172,10 +18172,10 @@ lean_dec(x_454); lean_dec_ref(x_453); lean_dec(x_452); lean_dec_ref(x_451); -x_17 = x_466; -x_18 = x_502; -x_19 = x_482; -x_20 = x_461; +x_17 = x_461; +x_18 = x_466; +x_19 = x_502; +x_20 = x_482; x_21 = x_450; x_22 = lean_box(0); goto block_47; @@ -18214,10 +18214,10 @@ lean_dec(x_454); lean_dec_ref(x_453); lean_dec(x_452); lean_dec_ref(x_517); -x_17 = x_466; -x_18 = x_502; -x_19 = x_482; -x_20 = x_461; +x_17 = x_461; +x_18 = x_466; +x_19 = x_502; +x_20 = x_482; x_21 = x_450; x_22 = lean_box(0); goto block_47; @@ -18417,7 +18417,7 @@ lean_dec_ref(x_453); lean_dec(x_452); lean_dec_ref(x_451); lean_dec(x_450); -lean_dec_ref(x_445); +lean_dec_ref(x_446); lean_dec(x_434); lean_dec(x_54); x_536 = lean_ctor_get(x_481, 0); @@ -18448,7 +18448,7 @@ lean_dec_ref(x_453); lean_dec(x_452); lean_dec_ref(x_451); lean_dec(x_450); -lean_dec_ref(x_445); +lean_dec_ref(x_446); lean_dec(x_434); lean_dec(x_54); x_539 = lean_ctor_get(x_476, 0); @@ -18475,8 +18475,8 @@ else lean_object* x_542; lean_object* x_543; lean_dec_ref(x_448); lean_dec_ref(x_447); -lean_dec(x_446); -lean_dec_ref(x_445); +lean_dec_ref(x_446); +lean_dec(x_445); lean_dec_ref(x_444); lean_dec_ref(x_443); lean_dec(x_441); @@ -18494,8 +18494,8 @@ else lean_object* x_544; lean_object* x_545; lean_dec_ref(x_448); lean_dec_ref(x_447); -lean_dec(x_446); -lean_dec_ref(x_445); +lean_dec_ref(x_446); +lean_dec(x_445); lean_dec_ref(x_444); lean_dec_ref(x_443); lean_dec(x_441); @@ -18577,12 +18577,12 @@ lean_dec(x_572); if (x_573 == 0) { lean_dec(x_570); -x_443 = x_560; -x_444 = x_561; -x_445 = x_568; -x_446 = x_569; -x_447 = x_555; -x_448 = x_559; +x_443 = x_561; +x_444 = x_559; +x_445 = x_569; +x_446 = x_568; +x_447 = x_560; +x_448 = x_555; x_449 = x_548; x_450 = x_549; x_451 = x_550; @@ -18608,12 +18608,12 @@ lean_ctor_set(x_576, 0, x_574); lean_ctor_set(x_576, 1, x_575); x_577 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_547, x_576, x_551, x_552, x_553); lean_dec_ref(x_577); -x_443 = x_560; -x_444 = x_561; -x_445 = x_568; -x_446 = x_569; -x_447 = x_555; -x_448 = x_559; +x_443 = x_561; +x_444 = x_559; +x_445 = x_569; +x_446 = x_568; +x_447 = x_560; +x_448 = x_555; x_449 = x_548; x_450 = x_549; x_451 = x_550; @@ -19021,27 +19021,27 @@ goto block_780; block_742: { uint8_t x_652; -x_652 = l_Lean_Expr_hasLooseBVars(x_641); +x_652 = l_Lean_Expr_hasLooseBVars(x_642); if (x_652 == 0) { uint8_t x_653; -x_653 = l_Lean_Expr_hasFVar(x_641); +x_653 = l_Lean_Expr_hasFVar(x_642); if (x_653 == 0) { lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; size_t x_658; size_t x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; -x_654 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_641, x_650); +x_654 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_642, x_650); x_655 = lean_ctor_get(x_654, 0); lean_inc(x_655); lean_dec_ref(x_654); x_656 = lean_box(0); -lean_inc(x_642); -x_657 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_642, x_656); -x_658 = lean_array_size(x_639); +lean_inc(x_641); +x_657 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_641, x_656); +x_658 = lean_array_size(x_643); x_659 = 0; -lean_inc_ref(x_639); -x_660 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_658, x_659, x_639); -x_661 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_643, x_50); -lean_dec_ref(x_643); +lean_inc_ref(x_643); +x_660 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_658, x_659, x_643); +x_661 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_644, x_50); +lean_dec_ref(x_644); x_662 = l_Array_append___redArg(x_660, x_661); lean_dec_ref(x_661); if (lean_obj_tag(x_655) == 1) @@ -19050,9 +19050,9 @@ lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_dec_ref(x_647); lean_dec(x_646); lean_dec_ref(x_645); -lean_dec_ref(x_644); -lean_dec(x_642); -lean_dec_ref(x_641); +lean_dec_ref(x_643); +lean_dec_ref(x_642); +lean_dec(x_641); lean_dec_ref(x_640); lean_dec_ref(x_639); lean_dec(x_637); @@ -19074,9 +19074,9 @@ if (x_667 == 0) lean_dec(x_650); lean_dec_ref(x_649); lean_dec(x_648); -x_9 = x_662; -x_10 = x_663; -x_11 = x_657; +x_9 = x_657; +x_10 = x_662; +x_11 = x_663; x_12 = lean_box(0); goto block_16; } @@ -19094,9 +19094,9 @@ lean_dec(x_650); lean_dec_ref(x_649); lean_dec(x_648); lean_dec_ref(x_671); -x_9 = x_662; -x_10 = x_663; -x_11 = x_657; +x_9 = x_657; +x_10 = x_662; +x_11 = x_663; x_12 = lean_box(0); goto block_16; } @@ -19109,7 +19109,7 @@ lean_inc(x_650); lean_inc_ref(x_649); lean_inc(x_648); lean_inc_ref(x_647); -x_672 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_637, x_49, x_644, x_639, x_640, x_642, x_645, x_646, x_647, x_648, x_649, x_650); +x_672 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_637, x_49, x_640, x_643, x_639, x_641, x_645, x_646, x_647, x_648, x_649, x_650); if (lean_obj_tag(x_672) == 0) { lean_object* x_673; size_t x_674; uint8_t x_675; uint8_t x_676; lean_object* x_677; @@ -19129,7 +19129,7 @@ lean_inc(x_678); lean_dec_ref(x_677); x_679 = lean_ctor_get(x_673, 0); lean_inc(x_679); -x_680 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_641, x_679, x_650); +x_680 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_642, x_679, x_650); lean_dec_ref(x_680); lean_inc(x_673); x_681 = l_Lean_Compiler_LCNF_Decl_saveBase___redArg(x_673, x_650); @@ -19209,10 +19209,10 @@ lean_dec(x_650); lean_dec_ref(x_649); lean_dec(x_648); lean_dec_ref(x_647); -x_17 = x_662; -x_18 = x_698; -x_19 = x_678; -x_20 = x_657; +x_17 = x_657; +x_18 = x_662; +x_19 = x_698; +x_20 = x_678; x_21 = x_646; x_22 = lean_box(0); goto block_47; @@ -19251,10 +19251,10 @@ lean_dec(x_650); lean_dec_ref(x_649); lean_dec(x_648); lean_dec_ref(x_713); -x_17 = x_662; -x_18 = x_698; -x_19 = x_678; -x_20 = x_657; +x_17 = x_657; +x_18 = x_662; +x_19 = x_698; +x_20 = x_678; x_21 = x_646; x_22 = lean_box(0); goto block_47; @@ -19454,7 +19454,7 @@ lean_dec_ref(x_649); lean_dec(x_648); lean_dec_ref(x_647); lean_dec(x_646); -lean_dec_ref(x_641); +lean_dec_ref(x_642); lean_dec(x_629); lean_dec(x_54); x_732 = lean_ctor_get(x_677, 0); @@ -19485,7 +19485,7 @@ lean_dec_ref(x_649); lean_dec(x_648); lean_dec_ref(x_647); lean_dec(x_646); -lean_dec_ref(x_641); +lean_dec_ref(x_642); lean_dec(x_629); lean_dec(x_54); x_735 = lean_ctor_get(x_672, 0); @@ -19512,8 +19512,8 @@ else lean_object* x_738; lean_object* x_739; lean_dec_ref(x_644); lean_dec_ref(x_643); -lean_dec(x_642); -lean_dec_ref(x_641); +lean_dec_ref(x_642); +lean_dec(x_641); lean_dec_ref(x_640); lean_dec_ref(x_639); lean_dec(x_637); @@ -19531,8 +19531,8 @@ else lean_object* x_740; lean_object* x_741; lean_dec_ref(x_644); lean_dec_ref(x_643); -lean_dec(x_642); -lean_dec_ref(x_641); +lean_dec_ref(x_642); +lean_dec(x_641); lean_dec_ref(x_640); lean_dec_ref(x_639); lean_dec(x_637); @@ -19614,12 +19614,12 @@ lean_dec(x_768); if (x_769 == 0) { lean_dec(x_766); -x_639 = x_756; -x_640 = x_757; -x_641 = x_764; -x_642 = x_765; -x_643 = x_751; -x_644 = x_755; +x_639 = x_757; +x_640 = x_755; +x_641 = x_765; +x_642 = x_764; +x_643 = x_756; +x_644 = x_751; x_645 = x_744; x_646 = x_745; x_647 = x_746; @@ -19645,12 +19645,12 @@ lean_ctor_set(x_772, 0, x_770); lean_ctor_set(x_772, 1, x_771); x_773 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_743, x_772, x_747, x_748, x_749); lean_dec_ref(x_773); -x_639 = x_756; -x_640 = x_757; -x_641 = x_764; -x_642 = x_765; -x_643 = x_751; -x_644 = x_755; +x_639 = x_757; +x_640 = x_755; +x_641 = x_765; +x_642 = x_764; +x_643 = x_756; +x_644 = x_751; x_645 = x_744; x_646 = x_745; x_647 = x_746; @@ -20095,27 +20095,27 @@ goto block_982; block_944: { uint8_t x_854; -x_854 = l_Lean_Expr_hasLooseBVars(x_843); +x_854 = l_Lean_Expr_hasLooseBVars(x_844); if (x_854 == 0) { uint8_t x_855; -x_855 = l_Lean_Expr_hasFVar(x_843); +x_855 = l_Lean_Expr_hasFVar(x_844); if (x_855 == 0) { lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; size_t x_860; size_t x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; -x_856 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_843, x_852); +x_856 = l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___redArg(x_844, x_852); x_857 = lean_ctor_get(x_856, 0); lean_inc(x_857); lean_dec_ref(x_856); x_858 = lean_box(0); -lean_inc(x_844); -x_859 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_844, x_858); -x_860 = lean_array_size(x_841); +lean_inc(x_843); +x_859 = l_List_mapTR_loop___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__1(x_843, x_858); +x_860 = lean_array_size(x_845); x_861 = 0; -lean_inc_ref(x_841); -x_862 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_860, x_861, x_841); -x_863 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_845, x_50); -lean_dec_ref(x_845); +lean_inc_ref(x_845); +x_862 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__2(x_860, x_861, x_845); +x_863 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_getRemainingArgs(x_846, x_50); +lean_dec_ref(x_846); x_864 = l_Array_append___redArg(x_862, x_863); lean_dec_ref(x_863); if (lean_obj_tag(x_857) == 1) @@ -20124,9 +20124,9 @@ lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; lean_dec_ref(x_849); lean_dec(x_848); lean_dec_ref(x_847); -lean_dec_ref(x_846); -lean_dec(x_844); -lean_dec_ref(x_843); +lean_dec_ref(x_845); +lean_dec_ref(x_844); +lean_dec(x_843); lean_dec_ref(x_842); lean_dec_ref(x_841); lean_dec(x_839); @@ -20148,9 +20148,9 @@ if (x_869 == 0) lean_dec(x_852); lean_dec_ref(x_851); lean_dec(x_850); -x_9 = x_864; -x_10 = x_865; -x_11 = x_859; +x_9 = x_859; +x_10 = x_864; +x_11 = x_865; x_12 = lean_box(0); goto block_16; } @@ -20168,9 +20168,9 @@ lean_dec(x_852); lean_dec_ref(x_851); lean_dec(x_850); lean_dec_ref(x_873); -x_9 = x_864; -x_10 = x_865; -x_11 = x_859; +x_9 = x_859; +x_10 = x_864; +x_11 = x_865; x_12 = lean_box(0); goto block_16; } @@ -20183,7 +20183,7 @@ lean_inc(x_852); lean_inc_ref(x_851); lean_inc(x_850); lean_inc_ref(x_849); -x_874 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_839, x_49, x_846, x_841, x_842, x_844, x_847, x_848, x_849, x_850, x_851, x_852); +x_874 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_mkSpecDecl(x_839, x_49, x_842, x_845, x_841, x_843, x_847, x_848, x_849, x_850, x_851, x_852); if (lean_obj_tag(x_874) == 0) { lean_object* x_875; size_t x_876; uint8_t x_877; uint8_t x_878; lean_object* x_879; @@ -20203,7 +20203,7 @@ lean_inc(x_880); lean_dec_ref(x_879); x_881 = lean_ctor_get(x_875, 0); lean_inc(x_881); -x_882 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_843, x_881, x_852); +x_882 = l_Lean_Compiler_LCNF_Specialize_cacheSpec___redArg(x_844, x_881, x_852); lean_dec_ref(x_882); lean_inc(x_875); x_883 = l_Lean_Compiler_LCNF_Decl_saveBase___redArg(x_875, x_852); @@ -20283,10 +20283,10 @@ lean_dec(x_852); lean_dec_ref(x_851); lean_dec(x_850); lean_dec_ref(x_849); -x_17 = x_864; -x_18 = x_900; -x_19 = x_880; -x_20 = x_859; +x_17 = x_859; +x_18 = x_864; +x_19 = x_900; +x_20 = x_880; x_21 = x_848; x_22 = lean_box(0); goto block_47; @@ -20325,10 +20325,10 @@ lean_dec(x_852); lean_dec_ref(x_851); lean_dec(x_850); lean_dec_ref(x_915); -x_17 = x_864; -x_18 = x_900; -x_19 = x_880; -x_20 = x_859; +x_17 = x_859; +x_18 = x_864; +x_19 = x_900; +x_20 = x_880; x_21 = x_848; x_22 = lean_box(0); goto block_47; @@ -20528,7 +20528,7 @@ lean_dec_ref(x_851); lean_dec(x_850); lean_dec_ref(x_849); lean_dec(x_848); -lean_dec_ref(x_843); +lean_dec_ref(x_844); lean_dec(x_831); lean_dec(x_824); x_934 = lean_ctor_get(x_879, 0); @@ -20559,7 +20559,7 @@ lean_dec_ref(x_851); lean_dec(x_850); lean_dec_ref(x_849); lean_dec(x_848); -lean_dec_ref(x_843); +lean_dec_ref(x_844); lean_dec(x_831); lean_dec(x_824); x_937 = lean_ctor_get(x_874, 0); @@ -20586,8 +20586,8 @@ else lean_object* x_940; lean_object* x_941; lean_dec_ref(x_846); lean_dec_ref(x_845); -lean_dec(x_844); -lean_dec_ref(x_843); +lean_dec_ref(x_844); +lean_dec(x_843); lean_dec_ref(x_842); lean_dec_ref(x_841); lean_dec(x_839); @@ -20605,8 +20605,8 @@ else lean_object* x_942; lean_object* x_943; lean_dec_ref(x_846); lean_dec_ref(x_845); -lean_dec(x_844); -lean_dec_ref(x_843); +lean_dec_ref(x_844); +lean_dec(x_843); lean_dec_ref(x_842); lean_dec_ref(x_841); lean_dec(x_839); @@ -20688,12 +20688,12 @@ lean_dec(x_970); if (x_971 == 0) { lean_dec(x_968); -x_841 = x_958; -x_842 = x_959; -x_843 = x_966; -x_844 = x_967; -x_845 = x_953; -x_846 = x_957; +x_841 = x_959; +x_842 = x_957; +x_843 = x_967; +x_844 = x_966; +x_845 = x_958; +x_846 = x_953; x_847 = x_946; x_848 = x_947; x_849 = x_948; @@ -20719,12 +20719,12 @@ lean_ctor_set(x_974, 0, x_972); lean_ctor_set(x_974, 1, x_973); x_975 = l_Lean_addTrace___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__4___redArg(x_945, x_974, x_949, x_950, x_951); lean_dec_ref(x_975); -x_841 = x_958; -x_842 = x_959; -x_843 = x_966; -x_844 = x_967; -x_845 = x_953; -x_846 = x_957; +x_841 = x_959; +x_842 = x_957; +x_843 = x_967; +x_844 = x_966; +x_845 = x_958; +x_846 = x_953; x_847 = x_946; x_848 = x_947; x_849 = x_948; @@ -21042,9 +21042,9 @@ return x_1033; { lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_alloc_ctor(3, 3, 0); -lean_ctor_set(x_13, 0, x_10); -lean_ctor_set(x_13, 1, x_11); -lean_ctor_set(x_13, 2, x_9); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_9); +lean_ctor_set(x_13, 2, x_10); x_14 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_14, 0, x_13); x_15 = lean_alloc_ctor(0, 1, 0); @@ -21061,19 +21061,19 @@ if (x_24 == 0) lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; x_25 = lean_ctor_get(x_23, 1); x_26 = lean_ctor_get(x_23, 3); -x_27 = lean_ctor_get(x_18, 0); +x_27 = lean_ctor_get(x_19, 0); lean_inc(x_27); -x_28 = lean_array_push(x_25, x_18); +x_28 = lean_array_push(x_25, x_19); lean_inc(x_27); -x_29 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__6___redArg(x_26, x_27, x_19); +x_29 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__6___redArg(x_26, x_27, x_20); lean_ctor_set(x_23, 3, x_29); lean_ctor_set(x_23, 1, x_28); x_30 = lean_st_ref_set(x_21, x_23); lean_dec(x_21); x_31 = lean_alloc_ctor(3, 3, 0); lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_20); -lean_ctor_set(x_31, 2, x_17); +lean_ctor_set(x_31, 1, x_17); +lean_ctor_set(x_31, 2, x_18); x_32 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_32, 0, x_31); x_33 = lean_alloc_ctor(0, 1, 0); @@ -21093,11 +21093,11 @@ lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); lean_dec(x_23); -x_39 = lean_ctor_get(x_18, 0); +x_39 = lean_ctor_get(x_19, 0); lean_inc(x_39); -x_40 = lean_array_push(x_35, x_18); +x_40 = lean_array_push(x_35, x_19); lean_inc(x_39); -x_41 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__6___redArg(x_37, x_39, x_19); +x_41 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__6___redArg(x_37, x_39, x_20); x_42 = lean_alloc_ctor(0, 4, 1); lean_ctor_set(x_42, 0, x_34); lean_ctor_set(x_42, 1, x_40); @@ -21108,8 +21108,8 @@ x_43 = lean_st_ref_set(x_21, x_42); lean_dec(x_21); x_44 = lean_alloc_ctor(3, 3, 0); lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_20); -lean_ctor_set(x_44, 2, x_17); +lean_ctor_set(x_44, 1, x_17); +lean_ctor_set(x_44, 2, x_18); x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_44); x_46 = lean_alloc_ctor(0, 1, 0); @@ -22253,7 +22253,7 @@ lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_55; uint8_t x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; 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_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_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +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_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; 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_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_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; x_17 = lean_ctor_get(x_1, 0); x_18 = lean_ctor_get(x_1, 1); x_149 = lean_ctor_get(x_17, 0); @@ -22468,12 +22468,12 @@ return x_184; { lean_object* x_30; lean_object* x_31; x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_22); -lean_ctor_set(x_30, 1, x_24); +lean_ctor_set(x_30, 0, x_27); +lean_ctor_set(x_30, 1, x_23); lean_ctor_set(x_30, 2, x_29); -lean_ctor_set(x_30, 3, x_26); +lean_ctor_set(x_30, 3, x_25); lean_inc_ref(x_18); -x_31 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_visitCode(x_18, x_30, x_27, x_20, x_23, x_21, x_28); +x_31 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_visitCode(x_18, x_30, x_21, x_26, x_19, x_22, x_20); if (lean_obj_tag(x_31) == 0) { lean_object* x_32; size_t x_33; size_t x_34; uint8_t x_35; @@ -22485,9 +22485,9 @@ x_34 = lean_ptr_addr(x_32); x_35 = lean_usize_dec_eq(x_33, x_34); if (x_35 == 0) { -x_9 = x_19; +x_9 = x_32; x_10 = lean_box(0); -x_11 = x_32; +x_11 = x_24; x_12 = x_35; goto block_16; } @@ -22495,54 +22495,54 @@ else { size_t x_36; size_t x_37; uint8_t x_38; x_36 = lean_ptr_addr(x_17); -x_37 = lean_ptr_addr(x_19); +x_37 = lean_ptr_addr(x_24); x_38 = lean_usize_dec_eq(x_36, x_37); -x_9 = x_19; +x_9 = x_32; x_10 = lean_box(0); -x_11 = x_32; +x_11 = x_24; x_12 = x_38; goto block_16; } } else { -lean_dec_ref(x_19); +lean_dec_ref(x_24); lean_dec_ref(x_1); return x_31; } } block_54: { -if (x_42 == 0) +if (x_41 == 0) { -lean_dec(x_47); -x_19 = x_41; -x_20 = x_40; +lean_dec(x_46); +x_19 = x_40; +x_20 = x_42; x_21 = x_43; -x_22 = x_44; -x_23 = x_45; -x_24 = x_52; -x_25 = lean_box(0); -x_26 = x_49; -x_27 = x_50; -x_28 = x_51; -x_29 = x_48; +x_22 = x_45; +x_23 = x_52; +x_24 = x_47; +x_25 = x_48; +x_26 = x_50; +x_27 = x_49; +x_28 = lean_box(0); +x_29 = x_44; goto block_39; } else { lean_object* x_53; -x_53 = l_Lean_FVarIdSet_insert(x_48, x_47); -x_19 = x_41; -x_20 = x_40; +x_53 = l_Lean_FVarIdSet_insert(x_44, x_46); +x_19 = x_40; +x_20 = x_42; x_21 = x_43; -x_22 = x_44; -x_23 = x_45; -x_24 = x_52; -x_25 = lean_box(0); -x_26 = x_49; -x_27 = x_50; -x_28 = x_51; +x_22 = x_45; +x_23 = x_52; +x_24 = x_47; +x_25 = x_48; +x_26 = x_50; +x_27 = x_49; +x_28 = lean_box(0); x_29 = x_53; goto block_39; } @@ -22559,58 +22559,58 @@ lean_inc(x_68); x_69 = lean_ctor_get(x_59, 3); lean_inc(x_69); lean_dec_ref(x_59); -lean_inc(x_57); -x_70 = l_Lean_FVarIdSet_insert(x_66, x_57); -if (x_56 == 0) -{ -x_40 = x_61; -x_41 = x_55; -x_42 = x_58; -x_43 = x_63; -x_44 = x_70; -x_45 = x_62; -x_46 = lean_box(0); +lean_inc(x_56); +x_70 = l_Lean_FVarIdSet_insert(x_66, x_56); +if (x_55 == 0) +{ +x_40 = x_62; +x_41 = x_58; +x_42 = x_64; +x_43 = x_60; +x_44 = x_68; +x_45 = x_63; +x_46 = x_56; x_47 = x_57; -x_48 = x_68; -x_49 = x_69; -x_50 = x_60; -x_51 = x_64; +x_48 = x_69; +x_49 = x_70; +x_50 = x_61; +x_51 = lean_box(0); x_52 = x_67; goto block_54; } else { lean_object* x_71; -lean_inc(x_57); -x_71 = l_Lean_FVarIdSet_insert(x_67, x_57); -x_40 = x_61; -x_41 = x_55; -x_42 = x_58; -x_43 = x_63; -x_44 = x_70; -x_45 = x_62; -x_46 = lean_box(0); +lean_inc(x_56); +x_71 = l_Lean_FVarIdSet_insert(x_67, x_56); +x_40 = x_62; +x_41 = x_58; +x_42 = x_64; +x_43 = x_60; +x_44 = x_68; +x_45 = x_63; +x_46 = x_56; x_47 = x_57; -x_48 = x_68; -x_49 = x_69; -x_50 = x_60; -x_51 = x_64; +x_48 = x_69; +x_49 = x_70; +x_50 = x_61; +x_51 = lean_box(0); x_52 = x_71; goto block_54; } } block_111: { -switch (lean_obj_tag(x_76)) { +switch (lean_obj_tag(x_80)) { case 3: { lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_76, 0); +x_84 = lean_ctor_get(x_80, 0); lean_inc(x_84); -x_85 = lean_ctor_get(x_76, 2); +x_85 = lean_ctor_get(x_80, 2); lean_inc_ref(x_85); -lean_dec_ref(x_76); -x_86 = l_Lean_Compiler_LCNF_getDecl_x3f___redArg(x_84, x_75, x_77); +lean_dec_ref(x_80); +x_86 = l_Lean_Compiler_LCNF_getDecl_x3f___redArg(x_84, x_78, x_73); if (lean_obj_tag(x_86) == 0) { lean_object* x_87; @@ -22622,16 +22622,16 @@ if (lean_obj_tag(x_87) == 0) uint8_t x_88; lean_dec_ref(x_85); x_88 = 0; -x_55 = x_73; -x_56 = x_82; -x_57 = x_78; +x_55 = x_82; +x_56 = x_76; +x_57 = x_77; x_58 = x_88; -x_59 = x_80; +x_59 = x_75; x_60 = x_79; -x_61 = x_75; -x_62 = x_81; -x_63 = x_74; -x_64 = x_77; +x_61 = x_78; +x_62 = x_74; +x_63 = x_81; +x_64 = x_73; x_65 = lean_box(0); goto block_72; } @@ -22649,16 +22649,16 @@ lean_dec_ref(x_85); x_92 = lean_array_get_size(x_90); lean_dec_ref(x_90); x_93 = lean_nat_dec_lt(x_91, x_92); -x_55 = x_73; -x_56 = x_82; -x_57 = x_78; +x_55 = x_82; +x_56 = x_76; +x_57 = x_77; x_58 = x_93; -x_59 = x_80; +x_59 = x_75; x_60 = x_79; -x_61 = x_75; -x_62 = x_81; -x_63 = x_74; -x_64 = x_77; +x_61 = x_78; +x_62 = x_74; +x_63 = x_81; +x_64 = x_73; x_65 = lean_box(0); goto block_72; } @@ -22667,14 +22667,14 @@ else { uint8_t x_94; lean_dec_ref(x_85); -lean_dec(x_81); -lean_dec_ref(x_80); +lean_dec_ref(x_81); lean_dec(x_79); -lean_dec(x_78); -lean_dec(x_77); +lean_dec_ref(x_78); +lean_dec_ref(x_77); +lean_dec(x_76); lean_dec_ref(x_75); -lean_dec_ref(x_74); -lean_dec_ref(x_73); +lean_dec(x_74); +lean_dec(x_73); lean_dec_ref(x_1); x_94 = !lean_is_exclusive(x_86); if (x_94 == 0) @@ -22696,12 +22696,12 @@ return x_96; case 4: { lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_76, 0); +x_97 = lean_ctor_get(x_80, 0); lean_inc(x_97); -x_98 = lean_ctor_get(x_76, 1); +x_98 = lean_ctor_get(x_80, 1); lean_inc_ref(x_98); -lean_dec_ref(x_76); -x_99 = l_Lean_Compiler_LCNF_findFunDecl_x3f___redArg(x_97, x_81); +lean_dec_ref(x_80); +x_99 = l_Lean_Compiler_LCNF_findFunDecl_x3f___redArg(x_97, x_74); lean_dec(x_97); if (lean_obj_tag(x_99) == 0) { @@ -22714,16 +22714,16 @@ if (lean_obj_tag(x_100) == 0) uint8_t x_101; lean_dec_ref(x_98); x_101 = 0; -x_55 = x_73; -x_56 = x_82; -x_57 = x_78; +x_55 = x_82; +x_56 = x_76; +x_57 = x_77; x_58 = x_101; -x_59 = x_80; +x_59 = x_75; x_60 = x_79; -x_61 = x_75; -x_62 = x_81; -x_63 = x_74; -x_64 = x_77; +x_61 = x_78; +x_62 = x_74; +x_63 = x_81; +x_64 = x_73; x_65 = lean_box(0); goto block_72; } @@ -22741,16 +22741,16 @@ lean_dec_ref(x_98); x_105 = lean_array_get_size(x_103); lean_dec_ref(x_103); x_106 = lean_nat_dec_lt(x_104, x_105); -x_55 = x_73; -x_56 = x_82; -x_57 = x_78; +x_55 = x_82; +x_56 = x_76; +x_57 = x_77; x_58 = x_106; -x_59 = x_80; +x_59 = x_75; x_60 = x_79; -x_61 = x_75; -x_62 = x_81; -x_63 = x_74; -x_64 = x_77; +x_61 = x_78; +x_62 = x_74; +x_63 = x_81; +x_64 = x_73; x_65 = lean_box(0); goto block_72; } @@ -22759,14 +22759,14 @@ else { uint8_t x_107; lean_dec_ref(x_98); -lean_dec(x_81); -lean_dec_ref(x_80); +lean_dec_ref(x_81); lean_dec(x_79); -lean_dec(x_78); -lean_dec(x_77); +lean_dec_ref(x_78); +lean_dec_ref(x_77); +lean_dec(x_76); lean_dec_ref(x_75); -lean_dec_ref(x_74); -lean_dec_ref(x_73); +lean_dec(x_74); +lean_dec(x_73); lean_dec_ref(x_1); x_107 = !lean_is_exclusive(x_99); if (x_107 == 0) @@ -22788,18 +22788,18 @@ return x_109; default: { uint8_t x_110; -lean_dec(x_76); +lean_dec(x_80); x_110 = 0; -x_55 = x_73; -x_56 = x_82; -x_57 = x_78; +x_55 = x_82; +x_56 = x_76; +x_57 = x_77; x_58 = x_110; -x_59 = x_80; +x_59 = x_75; x_60 = x_79; -x_61 = x_75; -x_62 = x_81; -x_63 = x_74; -x_64 = x_77; +x_61 = x_78; +x_62 = x_74; +x_63 = x_81; +x_64 = x_73; x_65 = lean_box(0); goto block_72; } @@ -22816,13 +22816,13 @@ lean_dec_ref(x_121); x_123 = lean_unbox(x_122); lean_dec(x_122); x_73 = x_112; -x_74 = x_113; -x_75 = x_114; +x_74 = x_114; +x_75 = x_113; x_76 = x_115; -x_77 = x_117; -x_78 = x_116; -x_79 = x_118; -x_80 = x_119; +x_77 = x_116; +x_78 = x_117; +x_79 = x_119; +x_80 = x_118; x_81 = x_120; x_82 = x_123; x_83 = lean_box(0); @@ -22831,15 +22831,15 @@ goto block_111; else { uint8_t x_124; -lean_dec(x_120); -lean_dec_ref(x_119); +lean_dec_ref(x_120); +lean_dec(x_119); lean_dec(x_118); -lean_dec(x_117); -lean_dec(x_116); +lean_dec_ref(x_117); +lean_dec_ref(x_116); lean_dec(x_115); -lean_dec_ref(x_114); +lean_dec(x_114); lean_dec_ref(x_113); -lean_dec_ref(x_112); +lean_dec(x_112); lean_dec_ref(x_1); x_124 = !lean_is_exclusive(x_121); if (x_124 == 0) @@ -22882,15 +22882,15 @@ if (x_143 == 0) { if (lean_obj_tag(x_140) == 0) { -x_112 = x_128; -x_113 = x_136; -x_114 = x_134; -x_115 = x_131; -x_116 = x_129; -x_117 = x_137; -x_118 = x_133; -x_119 = x_132; -x_120 = x_135; +x_112 = x_137; +x_113 = x_132; +x_114 = x_135; +x_115 = x_129; +x_116 = x_128; +x_117 = x_134; +x_118 = x_131; +x_119 = x_133; +x_120 = x_136; x_121 = x_141; goto block_127; } @@ -22900,15 +22900,15 @@ uint8_t x_144; lean_dec_ref(x_141); lean_dec_ref(x_140); x_144 = 1; -x_73 = x_128; -x_74 = x_136; -x_75 = x_134; -x_76 = x_131; -x_77 = x_137; -x_78 = x_129; +x_73 = x_137; +x_74 = x_135; +x_75 = x_132; +x_76 = x_129; +x_77 = x_128; +x_78 = x_134; x_79 = x_133; -x_80 = x_132; -x_81 = x_135; +x_80 = x_131; +x_81 = x_136; x_82 = x_144; x_83 = lean_box(0); goto block_111; @@ -22917,15 +22917,15 @@ goto block_111; else { lean_dec(x_140); -x_112 = x_128; -x_113 = x_136; -x_114 = x_134; -x_115 = x_131; -x_116 = x_129; -x_117 = x_137; -x_118 = x_133; -x_119 = x_132; -x_120 = x_135; +x_112 = x_137; +x_113 = x_132; +x_114 = x_135; +x_115 = x_129; +x_116 = x_128; +x_117 = x_134; +x_118 = x_131; +x_119 = x_133; +x_120 = x_136; x_121 = x_141; goto block_127; } @@ -22933,15 +22933,15 @@ goto block_127; else { lean_dec(x_140); -x_112 = x_128; -x_113 = x_136; -x_114 = x_134; -x_115 = x_131; -x_116 = x_129; -x_117 = x_137; -x_118 = x_133; -x_119 = x_132; -x_120 = x_135; +x_112 = x_137; +x_113 = x_132; +x_114 = x_135; +x_115 = x_129; +x_116 = x_128; +x_117 = x_134; +x_118 = x_131; +x_119 = x_133; +x_120 = x_136; x_121 = x_141; goto block_127; } @@ -23057,7 +23057,7 @@ x_194 = lean_ctor_get(x_1, 1); lean_dec(x_194); x_195 = lean_ctor_get(x_1, 0); lean_dec(x_195); -lean_ctor_set(x_1, 1, x_190); +lean_ctor_set(x_1, 1, x_191); lean_ctor_set(x_1, 0, x_188); if (lean_is_scalar(x_189)) { x_196 = lean_alloc_ctor(0, 1, 0); @@ -23073,7 +23073,7 @@ lean_object* x_197; lean_object* x_198; lean_dec(x_1); x_197 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_197, 0, x_188); -lean_ctor_set(x_197, 1, x_190); +lean_ctor_set(x_197, 1, x_191); if (lean_is_scalar(x_189)) { x_198 = lean_alloc_ctor(0, 1, 0); } else { @@ -23086,7 +23086,7 @@ return x_198; else { lean_object* x_199; -lean_dec_ref(x_190); +lean_dec_ref(x_191); lean_dec(x_188); if (lean_is_scalar(x_189)) { x_199 = lean_alloc_ctor(0, 1, 0); @@ -23122,8 +23122,8 @@ x_216 = lean_ptr_addr(x_214); x_217 = lean_usize_dec_eq(x_215, x_216); if (x_217 == 0) { -x_190 = x_214; -x_191 = lean_box(0); +x_190 = lean_box(0); +x_191 = x_214; x_192 = x_217; goto block_200; } @@ -23133,8 +23133,8 @@ size_t x_218; size_t x_219; uint8_t x_220; x_218 = lean_ptr_addr(x_185); x_219 = lean_ptr_addr(x_188); x_220 = lean_usize_dec_eq(x_218, x_219); -x_190 = x_214; -x_191 = lean_box(0); +x_190 = lean_box(0); +x_191 = x_214; x_192 = x_220; goto block_200; } @@ -23682,8 +23682,8 @@ if (x_12 == 0) lean_object* x_13; lean_object* x_14; lean_dec_ref(x_1); x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_9); -lean_ctor_set(x_13, 1, x_11); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_9); x_14 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_14, 0, x_13); return x_14; @@ -24107,7 +24107,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeDecl(lean_object* x_1, 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_9; lean_object* x_10; lean_object* x_11; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_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_195; lean_object* x_196; uint8_t x_197; +uint8_t x_9; lean_object* x_10; lean_object* x_11; 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_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_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_195; lean_object* x_196; uint8_t x_197; x_16 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f___closed__2; x_195 = l_Lean_isTracingEnabledFor___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeApp_x3f_spec__3___redArg(x_16, x_6); x_196 = lean_ctor_get(x_195, 0); @@ -24173,8 +24173,8 @@ lean_dec(x_23); lean_dec_ref(x_22); lean_dec(x_21); lean_dec_ref(x_20); -lean_dec(x_17); -x_9 = x_18; +lean_dec(x_18); +x_9 = x_17; x_10 = x_19; x_11 = lean_box(0); goto block_15; @@ -24194,7 +24194,7 @@ x_29 = lean_ctor_get(x_28, 0); lean_inc(x_29); lean_dec_ref(x_28); x_30 = l___private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeDecl___closed__1; -x_31 = l_Lean_MessageData_ofName(x_17); +x_31 = l_Lean_MessageData_ofName(x_18); x_32 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); @@ -24211,7 +24211,7 @@ lean_dec(x_23); lean_dec_ref(x_22); lean_dec(x_21); lean_dec_ref(x_37); -x_9 = x_18; +x_9 = x_17; x_10 = x_19; x_11 = lean_box(0); goto block_15; @@ -24223,7 +24223,7 @@ lean_dec(x_23); lean_dec_ref(x_22); lean_dec(x_21); lean_dec_ref(x_19); -lean_dec(x_17); +lean_dec(x_18); x_38 = !lean_is_exclusive(x_28); if (x_38 == 0) { @@ -24247,44 +24247,44 @@ return x_40; lean_object* x_63; lean_object* x_64; x_63 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_51); -lean_ctor_set(x_63, 2, x_52); -lean_ctor_set(x_63, 3, x_53); -lean_inc(x_59); -lean_inc_ref(x_55); +lean_ctor_set(x_63, 1, x_49); +lean_ctor_set(x_63, 2, x_50); +lean_ctor_set(x_63, 3, x_51); +lean_inc(x_55); +lean_inc_ref(x_59); lean_inc(x_58); -lean_inc_ref(x_57); -lean_inc(x_43); -x_64 = l_Lean_Compiler_LCNF_DeclValue_mapCodeM___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeDecl_spec__0(x_46, x_50, x_63, x_43, x_57, x_58, x_55, x_59); +lean_inc_ref(x_42); +lean_inc(x_53); +x_64 = l_Lean_Compiler_LCNF_DeclValue_mapCodeM___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_specializeDecl_spec__0(x_52, x_45, x_63, x_53, x_42, x_58, x_59, x_55); if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); lean_dec_ref(x_64); -x_66 = lean_st_ref_get(x_43); -lean_dec(x_43); +x_66 = lean_st_ref_get(x_53); +lean_dec(x_53); x_67 = lean_ctor_get_uint8(x_66, sizeof(void*)*4); lean_dec(x_66); -lean_inc(x_56); +lean_inc(x_46); x_68 = lean_alloc_ctor(0, 6, 2); -lean_ctor_set(x_68, 0, x_56); -lean_ctor_set(x_68, 1, x_45); -lean_ctor_set(x_68, 2, x_61); -lean_ctor_set(x_68, 3, x_47); +lean_ctor_set(x_68, 0, x_46); +lean_ctor_set(x_68, 1, x_57); +lean_ctor_set(x_68, 2, x_44); +lean_ctor_set(x_68, 3, x_61); lean_ctor_set(x_68, 4, x_65); -lean_ctor_set(x_68, 5, x_49); -lean_ctor_set_uint8(x_68, sizeof(void*)*6, x_60); -lean_ctor_set_uint8(x_68, sizeof(void*)*6 + 1, x_48); +lean_ctor_set(x_68, 5, x_47); +lean_ctor_set_uint8(x_68, sizeof(void*)*6, x_48); +lean_ctor_set_uint8(x_68, sizeof(void*)*6 + 1, x_60); if (x_67 == 0) { -x_17 = x_56; -x_18 = x_67; +x_17 = x_67; +x_18 = x_46; x_19 = x_68; -x_20 = x_57; +x_20 = x_42; x_21 = x_58; -x_22 = x_55; -x_23 = x_59; +x_22 = x_59; +x_23 = x_55; x_24 = lean_box(0); goto block_41; } @@ -24295,36 +24295,36 @@ x_69 = lean_alloc_ctor(0, 0, 4); lean_ctor_set_uint8(x_69, 0, x_54); lean_ctor_set_uint8(x_69, 1, x_54); lean_ctor_set_uint8(x_69, 2, x_54); -lean_ctor_set_uint8(x_69, 3, x_44); -lean_inc(x_59); -lean_inc_ref(x_55); +lean_ctor_set_uint8(x_69, 3, x_56); +lean_inc(x_55); +lean_inc_ref(x_59); lean_inc(x_58); -lean_inc_ref(x_57); -x_70 = l_Lean_Compiler_LCNF_Decl_simp(x_68, x_69, x_57, x_58, x_55, x_59); +lean_inc_ref(x_42); +x_70 = l_Lean_Compiler_LCNF_Decl_simp(x_68, x_69, x_42, x_58, x_59, x_55); if (lean_obj_tag(x_70) == 0) { lean_object* x_71; x_71 = lean_ctor_get(x_70, 0); lean_inc(x_71); lean_dec_ref(x_70); -x_17 = x_56; -x_18 = x_67; +x_17 = x_67; +x_18 = x_46; x_19 = x_71; -x_20 = x_57; +x_20 = x_42; x_21 = x_58; -x_22 = x_55; -x_23 = x_59; +x_22 = x_59; +x_23 = x_55; x_24 = lean_box(0); goto block_41; } else { uint8_t x_72; -lean_dec(x_59); +lean_dec_ref(x_59); lean_dec(x_58); -lean_dec_ref(x_57); -lean_dec(x_56); -lean_dec_ref(x_55); +lean_dec(x_55); +lean_dec(x_46); +lean_dec_ref(x_42); x_72 = !lean_is_exclusive(x_70); if (x_72 == 0) { @@ -24347,15 +24347,15 @@ else { uint8_t x_75; lean_dec_ref(x_61); -lean_dec(x_59); +lean_dec_ref(x_59); lean_dec(x_58); -lean_dec_ref(x_57); -lean_dec(x_56); -lean_dec_ref(x_55); -lean_dec(x_49); -lean_dec_ref(x_47); -lean_dec(x_45); -lean_dec(x_43); +lean_dec(x_57); +lean_dec(x_55); +lean_dec(x_53); +lean_dec(x_47); +lean_dec(x_46); +lean_dec_ref(x_44); +lean_dec_ref(x_42); x_75 = !lean_is_exclusive(x_64); if (x_75 == 0) { @@ -24433,26 +24433,26 @@ if (x_110 == 0) uint8_t x_111; x_111 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_106; -x_45 = x_95; -x_46 = x_107; -x_47 = x_97; -x_48 = x_100; -x_49 = x_101; -x_50 = x_98; -x_51 = x_103; -x_52 = x_104; -x_53 = x_105; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_96; +x_45 = x_98; +x_46 = x_94; +x_47 = x_101; +x_48 = x_99; +x_49 = x_103; +x_50 = x_104; +x_51 = x_105; +x_52 = x_107; +x_53 = x_80; x_54 = x_111; -x_55 = x_83; -x_56 = x_94; -x_57 = x_81; +x_55 = x_84; +x_56 = x_106; +x_57 = x_95; x_58 = x_82; -x_59 = x_84; -x_60 = x_99; -x_61 = x_96; +x_59 = x_83; +x_60 = x_100; +x_61 = x_97; x_62 = x_102; goto block_78; } @@ -24465,26 +24465,26 @@ if (x_112 == 0) uint8_t x_113; x_113 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_106; -x_45 = x_95; -x_46 = x_107; -x_47 = x_97; -x_48 = x_100; -x_49 = x_101; -x_50 = x_98; -x_51 = x_103; -x_52 = x_104; -x_53 = x_105; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_96; +x_45 = x_98; +x_46 = x_94; +x_47 = x_101; +x_48 = x_99; +x_49 = x_103; +x_50 = x_104; +x_51 = x_105; +x_52 = x_107; +x_53 = x_80; x_54 = x_113; -x_55 = x_83; -x_56 = x_94; -x_57 = x_81; +x_55 = x_84; +x_56 = x_106; +x_57 = x_95; x_58 = x_82; -x_59 = x_84; -x_60 = x_99; -x_61 = x_96; +x_59 = x_83; +x_60 = x_100; +x_61 = x_97; x_62 = x_102; goto block_78; } @@ -24496,26 +24496,26 @@ x_115 = lean_usize_of_nat(x_109); x_116 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_visitFunDecl_spec__0(x_97, x_114, x_115, x_102); x_117 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_106; -x_45 = x_95; -x_46 = x_107; -x_47 = x_97; -x_48 = x_100; -x_49 = x_101; -x_50 = x_98; -x_51 = x_103; -x_52 = x_104; -x_53 = x_105; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_96; +x_45 = x_98; +x_46 = x_94; +x_47 = x_101; +x_48 = x_99; +x_49 = x_103; +x_50 = x_104; +x_51 = x_105; +x_52 = x_107; +x_53 = x_80; x_54 = x_117; -x_55 = x_83; -x_56 = x_94; -x_57 = x_81; +x_55 = x_84; +x_56 = x_106; +x_57 = x_95; x_58 = x_82; -x_59 = x_84; -x_60 = x_99; -x_61 = x_96; +x_59 = x_83; +x_60 = x_100; +x_61 = x_97; x_62 = x_116; goto block_78; } @@ -24575,26 +24575,26 @@ if (x_141 == 0) uint8_t x_142; x_142 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_137; -x_45 = x_126; -x_46 = x_138; -x_47 = x_128; -x_48 = x_131; -x_49 = x_132; -x_50 = x_129; -x_51 = x_134; -x_52 = x_135; -x_53 = x_136; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_127; +x_45 = x_129; +x_46 = x_125; +x_47 = x_132; +x_48 = x_130; +x_49 = x_134; +x_50 = x_135; +x_51 = x_136; +x_52 = x_138; +x_53 = x_80; x_54 = x_142; -x_55 = x_83; -x_56 = x_125; -x_57 = x_81; +x_55 = x_84; +x_56 = x_137; +x_57 = x_126; x_58 = x_82; -x_59 = x_84; -x_60 = x_130; -x_61 = x_127; +x_59 = x_83; +x_60 = x_131; +x_61 = x_128; x_62 = x_133; goto block_78; } @@ -24607,26 +24607,26 @@ if (x_143 == 0) uint8_t x_144; x_144 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_137; -x_45 = x_126; -x_46 = x_138; -x_47 = x_128; -x_48 = x_131; -x_49 = x_132; -x_50 = x_129; -x_51 = x_134; -x_52 = x_135; -x_53 = x_136; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_127; +x_45 = x_129; +x_46 = x_125; +x_47 = x_132; +x_48 = x_130; +x_49 = x_134; +x_50 = x_135; +x_51 = x_136; +x_52 = x_138; +x_53 = x_80; x_54 = x_144; -x_55 = x_83; -x_56 = x_125; -x_57 = x_81; +x_55 = x_84; +x_56 = x_137; +x_57 = x_126; x_58 = x_82; -x_59 = x_84; -x_60 = x_130; -x_61 = x_127; +x_59 = x_83; +x_60 = x_131; +x_61 = x_128; x_62 = x_133; goto block_78; } @@ -24638,26 +24638,26 @@ x_146 = lean_usize_of_nat(x_140); x_147 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_visitFunDecl_spec__0(x_128, x_145, x_146, x_133); x_148 = lean_unbox(x_88); lean_dec(x_88); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_137; -x_45 = x_126; -x_46 = x_138; -x_47 = x_128; -x_48 = x_131; -x_49 = x_132; -x_50 = x_129; -x_51 = x_134; -x_52 = x_135; -x_53 = x_136; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_127; +x_45 = x_129; +x_46 = x_125; +x_47 = x_132; +x_48 = x_130; +x_49 = x_134; +x_50 = x_135; +x_51 = x_136; +x_52 = x_138; +x_53 = x_80; x_54 = x_148; -x_55 = x_83; -x_56 = x_125; -x_57 = x_81; +x_55 = x_84; +x_56 = x_137; +x_57 = x_126; x_58 = x_82; -x_59 = x_84; -x_60 = x_130; -x_61 = x_127; +x_59 = x_83; +x_60 = x_131; +x_61 = x_128; x_62 = x_147; goto block_78; } @@ -24758,26 +24758,26 @@ if (x_179 == 0) uint8_t x_180; x_180 = lean_unbox(x_152); lean_dec(x_152); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_175; -x_45 = x_164; -x_46 = x_176; -x_47 = x_166; -x_48 = x_169; -x_49 = x_170; -x_50 = x_167; -x_51 = x_172; -x_52 = x_173; -x_53 = x_174; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_165; +x_45 = x_167; +x_46 = x_163; +x_47 = x_170; +x_48 = x_168; +x_49 = x_172; +x_50 = x_173; +x_51 = x_174; +x_52 = x_176; +x_53 = x_80; x_54 = x_180; -x_55 = x_83; -x_56 = x_163; -x_57 = x_81; +x_55 = x_84; +x_56 = x_175; +x_57 = x_164; x_58 = x_82; -x_59 = x_84; -x_60 = x_168; -x_61 = x_165; +x_59 = x_83; +x_60 = x_169; +x_61 = x_166; x_62 = x_171; goto block_78; } @@ -24790,26 +24790,26 @@ if (x_181 == 0) uint8_t x_182; x_182 = lean_unbox(x_152); lean_dec(x_152); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_175; -x_45 = x_164; -x_46 = x_176; -x_47 = x_166; -x_48 = x_169; -x_49 = x_170; -x_50 = x_167; -x_51 = x_172; -x_52 = x_173; -x_53 = x_174; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_165; +x_45 = x_167; +x_46 = x_163; +x_47 = x_170; +x_48 = x_168; +x_49 = x_172; +x_50 = x_173; +x_51 = x_174; +x_52 = x_176; +x_53 = x_80; x_54 = x_182; -x_55 = x_83; -x_56 = x_163; -x_57 = x_81; +x_55 = x_84; +x_56 = x_175; +x_57 = x_164; x_58 = x_82; -x_59 = x_84; -x_60 = x_168; -x_61 = x_165; +x_59 = x_83; +x_60 = x_169; +x_61 = x_166; x_62 = x_171; goto block_78; } @@ -24821,26 +24821,26 @@ x_184 = lean_usize_of_nat(x_178); x_185 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Compiler_LCNF_Specialize_0__Lean_Compiler_LCNF_Specialize_visitFunDecl_spec__0(x_166, x_183, x_184, x_171); x_186 = lean_unbox(x_152); lean_dec(x_152); -x_42 = lean_box(0); -x_43 = x_80; -x_44 = x_175; -x_45 = x_164; -x_46 = x_176; -x_47 = x_166; -x_48 = x_169; -x_49 = x_170; -x_50 = x_167; -x_51 = x_172; -x_52 = x_173; -x_53 = x_174; +x_42 = x_81; +x_43 = lean_box(0); +x_44 = x_165; +x_45 = x_167; +x_46 = x_163; +x_47 = x_170; +x_48 = x_168; +x_49 = x_172; +x_50 = x_173; +x_51 = x_174; +x_52 = x_176; +x_53 = x_80; x_54 = x_186; -x_55 = x_83; -x_56 = x_163; -x_57 = x_81; +x_55 = x_84; +x_56 = x_175; +x_57 = x_164; x_58 = x_82; -x_59 = x_84; -x_60 = x_168; -x_61 = x_165; +x_59 = x_83; +x_60 = x_169; +x_61 = x_166; x_62 = x_185; goto block_78; } diff --git a/stage0/stdlib/Lean/Data/Json/Basic.c b/stage0/stdlib/Lean/Data/Json/Basic.c index 6c109c14053c..4bf060017d6c 100644 --- a/stage0/stdlib/Lean/Data/Json/Basic.c +++ b/stage0/stdlib/Lean/Data/Json/Basic.c @@ -3209,9 +3209,9 @@ goto block_52; block_45: { lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_nat_add(x_40, x_41); +x_42 = lean_nat_add(x_39, x_41); lean_dec(x_41); -lean_dec(x_40); +lean_dec(x_39); if (lean_is_scalar(x_36)) { x_43 = lean_alloc_ctor(0, 5, 0); } else { @@ -3230,7 +3230,7 @@ if (lean_is_scalar(x_26)) { lean_ctor_set(x_44, 0, x_38); lean_ctor_set(x_44, 1, x_28); lean_ctor_set(x_44, 2, x_29); -lean_ctor_set(x_44, 3, x_39); +lean_ctor_set(x_44, 3, x_40); lean_ctor_set(x_44, 4, x_43); return x_44; } @@ -3256,8 +3256,8 @@ if (lean_obj_tag(x_31) == 0) lean_object* x_50; x_50 = lean_ctor_get(x_31, 0); lean_inc(x_50); -x_39 = x_48; -x_40 = x_49; +x_39 = x_49; +x_40 = x_48; x_41 = x_50; goto block_45; } @@ -3265,8 +3265,8 @@ else { lean_object* x_51; x_51 = lean_unsigned_to_nat(0u); -x_39 = x_48; -x_40 = x_49; +x_39 = x_49; +x_40 = x_48; x_41 = x_51; goto block_45; } @@ -3682,9 +3682,9 @@ goto block_152; block_144: { lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_141 = lean_nat_add(x_139, x_140); +x_141 = lean_nat_add(x_138, x_140); lean_dec(x_140); -lean_dec(x_139); +lean_dec(x_138); if (lean_is_scalar(x_135)) { x_142 = lean_alloc_ctor(0, 5, 0); } else { @@ -3703,7 +3703,7 @@ if (lean_is_scalar(x_125)) { lean_ctor_set(x_143, 0, x_137); lean_ctor_set(x_143, 1, x_128); lean_ctor_set(x_143, 2, x_129); -lean_ctor_set(x_143, 3, x_138); +lean_ctor_set(x_143, 3, x_139); lean_ctor_set(x_143, 4, x_142); return x_143; } @@ -3729,8 +3729,8 @@ if (lean_obj_tag(x_131) == 0) lean_object* x_150; x_150 = lean_ctor_get(x_131, 0); lean_inc(x_150); -x_138 = x_148; -x_139 = x_149; +x_138 = x_149; +x_139 = x_148; x_140 = x_150; goto block_144; } @@ -3738,8 +3738,8 @@ else { lean_object* x_151; x_151 = lean_unsigned_to_nat(0u); -x_138 = x_148; -x_139 = x_149; +x_138 = x_149; +x_139 = x_148; x_140 = x_151; goto block_144; } @@ -5178,9 +5178,9 @@ goto block_53; block_46: { lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_nat_add(x_41, x_42); +x_43 = lean_nat_add(x_40, x_42); lean_dec(x_42); -lean_dec(x_41); +lean_dec(x_40); if (lean_is_scalar(x_36)) { x_44 = lean_alloc_ctor(0, 5, 0); } else { @@ -5199,7 +5199,7 @@ if (lean_is_scalar(x_26)) { lean_ctor_set(x_45, 0, x_39); lean_ctor_set(x_45, 1, x_28); lean_ctor_set(x_45, 2, x_29); -lean_ctor_set(x_45, 3, x_40); +lean_ctor_set(x_45, 3, x_41); lean_ctor_set(x_45, 4, x_44); return x_45; } @@ -5225,8 +5225,8 @@ if (lean_obj_tag(x_31) == 0) lean_object* x_51; x_51 = lean_ctor_get(x_31, 0); lean_inc(x_51); -x_40 = x_49; -x_41 = x_50; +x_40 = x_50; +x_41 = x_49; x_42 = x_51; goto block_46; } @@ -5234,8 +5234,8 @@ else { lean_object* x_52; x_52 = lean_unsigned_to_nat(0u); -x_40 = x_49; -x_41 = x_50; +x_40 = x_50; +x_41 = x_49; x_42 = x_52; goto block_46; } @@ -5806,9 +5806,9 @@ goto block_190; block_182: { lean_object* x_179; lean_object* x_180; lean_object* x_181; -x_179 = lean_nat_add(x_176, x_178); +x_179 = lean_nat_add(x_177, x_178); lean_dec(x_178); -lean_dec(x_176); +lean_dec(x_177); if (lean_is_scalar(x_172)) { x_180 = lean_alloc_ctor(0, 5, 0); } else { @@ -5827,7 +5827,7 @@ if (lean_is_scalar(x_162)) { lean_ctor_set(x_181, 0, x_175); lean_ctor_set(x_181, 1, x_165); lean_ctor_set(x_181, 2, x_166); -lean_ctor_set(x_181, 3, x_177); +lean_ctor_set(x_181, 3, x_176); lean_ctor_set(x_181, 4, x_180); return x_181; } @@ -5853,8 +5853,8 @@ if (lean_obj_tag(x_168) == 0) lean_object* x_188; x_188 = lean_ctor_get(x_168, 0); lean_inc(x_188); -x_176 = x_187; -x_177 = x_186; +x_176 = x_186; +x_177 = x_187; x_178 = x_188; goto block_182; } @@ -5862,8 +5862,8 @@ else { lean_object* x_189; x_189 = lean_unsigned_to_nat(0u); -x_176 = x_187; -x_177 = x_186; +x_176 = x_186; +x_177 = x_187; x_178 = x_189; goto block_182; } diff --git a/stage0/stdlib/Lean/DocString/Add.c b/stage0/stdlib/Lean/DocString/Add.c index bd55d065fb08..0c2e483eb380 100644 --- a/stage0/stdlib/Lean/DocString/Add.c +++ b/stage0/stdlib/Lean/DocString/Add.c @@ -2869,26 +2869,26 @@ goto block_79; block_50: { 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_dec_ref(x_13); -x_24 = lean_st_ref_get(x_17); +lean_dec_ref(x_22); +x_24 = lean_st_ref_get(x_21); x_25 = lean_ctor_get(x_24, 0); lean_inc_ref(x_25); lean_dec(x_24); +lean_inc_ref(x_19); lean_inc_ref(x_14); -lean_inc_ref(x_11); x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_11); -lean_ctor_set(x_26, 1, x_10); -lean_ctor_set(x_26, 2, x_14); +lean_ctor_set(x_26, 0, x_14); +lean_ctor_set(x_26, 1, x_18); +lean_ctor_set(x_26, 2, x_19); lean_ctor_set(x_26, 3, x_23); lean_inc_ref(x_25); x_27 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_22); -lean_ctor_set(x_27, 2, x_19); -lean_ctor_set(x_27, 3, x_12); -x_28 = l_Lean_Parser_mkParserState(x_11); -lean_dec_ref(x_11); +lean_ctor_set(x_27, 1, x_9); +lean_ctor_set(x_27, 2, x_11); +lean_ctor_set(x_27, 3, x_10); +x_28 = l_Lean_Parser_mkParserState(x_14); +lean_dec_ref(x_14); x_29 = l_Lean_Parser_ParserState_setPos(x_28, x_15); x_30 = lean_box(0); x_31 = l_Lean_parseVersoDocString___redArg___lam__4___closed__1; @@ -2904,8 +2904,8 @@ lean_dec_ref(x_33); x_36 = lean_box(0); x_37 = lean_array_size(x_34); x_38 = 0; -x_39 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_parseVersoDocString___at___00Lean_versoDocString_spec__0_spec__0___redArg(x_14, x_36, x_35, x_34, x_37, x_38, x_36, x_18, x_17); -lean_dec_ref(x_18); +x_39 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_parseVersoDocString___at___00Lean_versoDocString_spec__0_spec__0___redArg(x_19, x_36, x_35, x_34, x_37, x_38, x_36, x_16, x_21); +lean_dec_ref(x_16); lean_dec_ref(x_34); if (lean_obj_tag(x_39) == 0) { @@ -2952,8 +2952,8 @@ else { lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_dec_ref(x_34); -lean_dec_ref(x_18); -lean_dec_ref(x_14); +lean_dec_ref(x_19); +lean_dec_ref(x_16); x_46 = lean_ctor_get(x_33, 0); lean_inc_ref(x_46); lean_dec_ref(x_33); @@ -3009,39 +3009,39 @@ x_74 = lean_nat_dec_le(x_72, x_73); if (x_74 == 0) { lean_dec(x_72); -x_9 = lean_box(0); -x_10 = x_58; -x_11 = x_70; -x_12 = x_62; -x_13 = x_51; -x_14 = x_59; +x_9 = x_60; +x_10 = x_62; +x_11 = x_61; +x_12 = x_52; +x_13 = x_53; +x_14 = x_70; x_15 = x_67; -x_16 = x_53; -x_17 = x_56; -x_18 = x_55; -x_19 = x_61; -x_20 = x_52; -x_21 = x_54; -x_22 = x_60; +x_16 = x_55; +x_17 = lean_box(0); +x_18 = x_58; +x_19 = x_59; +x_20 = x_54; +x_21 = x_56; +x_22 = x_51; x_23 = x_73; goto block_50; } else { -x_9 = lean_box(0); -x_10 = x_58; -x_11 = x_70; -x_12 = x_62; -x_13 = x_51; -x_14 = x_59; +x_9 = x_60; +x_10 = x_62; +x_11 = x_61; +x_12 = x_52; +x_13 = x_53; +x_14 = x_70; x_15 = x_67; -x_16 = x_53; -x_17 = x_56; -x_18 = x_55; -x_19 = x_61; -x_20 = x_52; -x_21 = x_54; -x_22 = x_60; +x_16 = x_55; +x_17 = lean_box(0); +x_18 = x_58; +x_19 = x_59; +x_20 = x_54; +x_21 = x_56; +x_22 = x_51; x_23 = x_72; goto block_50; } @@ -3862,7 +3862,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_versoDocStringFromString_spec__3___redArg(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) { _start: { -lean_object* x_10; uint8_t 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_50; uint8_t x_51; uint8_t x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_50; uint8_t x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -3899,13 +3899,13 @@ x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_10); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_14); -lean_ctor_set(x_27, 1, x_15); -lean_ctor_set(x_27, 2, x_12); -lean_ctor_set(x_27, 3, x_16); +lean_ctor_set(x_27, 0, x_15); +lean_ctor_set(x_27, 1, x_12); +lean_ctor_set(x_27, 2, x_16); +lean_ctor_set(x_27, 3, x_13); lean_ctor_set(x_27, 4, x_26); -lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_13); -lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_11); +lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_11); +lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_14); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); lean_ctor_set(x_20, 6, x_28); @@ -3944,13 +3944,13 @@ x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); lean_ctor_set(x_42, 1, x_10); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_14); -lean_ctor_set(x_43, 1, x_15); -lean_ctor_set(x_43, 2, x_12); -lean_ctor_set(x_43, 3, x_16); +lean_ctor_set(x_43, 0, x_15); +lean_ctor_set(x_43, 1, x_12); +lean_ctor_set(x_43, 2, x_16); +lean_ctor_set(x_43, 3, x_13); lean_ctor_set(x_43, 4, x_42); -lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_13); -lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_11); +lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_11); +lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_14); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); x_45 = lean_alloc_ctor(0, 9, 0); @@ -3980,25 +3980,25 @@ if (x_60 == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); -lean_inc_ref(x_56); -x_62 = l_Lean_FileMap_toPosition(x_56, x_55); -lean_dec(x_55); -x_63 = l_Lean_FileMap_toPosition(x_56, x_57); +lean_inc_ref(x_52); +x_62 = l_Lean_FileMap_toPosition(x_52, x_56); +lean_dec(x_56); +x_63 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); x_65 = l_Lean_parseVersoDocString___redArg___lam__2___closed__0; -if (x_52 == 0) +if (x_53 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); x_10 = x_61; x_11 = x_51; -x_12 = x_64; -x_13 = x_54; -x_14 = x_53; -x_15 = x_62; -x_16 = x_65; +x_12 = x_62; +x_13 = x_65; +x_14 = x_54; +x_15 = x_55; +x_16 = x_64; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -4015,7 +4015,7 @@ lean_object* x_67; lean_dec_ref(x_64); lean_dec_ref(x_62); lean_dec(x_61); -lean_dec_ref(x_53); +lean_dec_ref(x_55); lean_dec_ref(x_7); x_67 = lean_box(0); lean_ctor_set(x_59, 0, x_67); @@ -4026,11 +4026,11 @@ else lean_free_object(x_59); x_10 = x_61; x_11 = x_51; -x_12 = x_64; -x_13 = x_54; -x_14 = x_53; -x_15 = x_62; -x_16 = x_65; +x_12 = x_62; +x_13 = x_65; +x_14 = x_54; +x_15 = x_55; +x_16 = x_64; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -4044,24 +4044,24 @@ lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); -lean_inc_ref(x_56); -x_69 = l_Lean_FileMap_toPosition(x_56, x_55); -lean_dec(x_55); -x_70 = l_Lean_FileMap_toPosition(x_56, x_57); +lean_inc_ref(x_52); +x_69 = l_Lean_FileMap_toPosition(x_52, x_56); +lean_dec(x_56); +x_70 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); x_72 = l_Lean_parseVersoDocString___redArg___lam__2___closed__0; -if (x_52 == 0) +if (x_53 == 0) { lean_dec_ref(x_50); x_10 = x_68; x_11 = x_51; -x_12 = x_71; -x_13 = x_54; -x_14 = x_53; -x_15 = x_69; -x_16 = x_72; +x_12 = x_69; +x_13 = x_72; +x_14 = x_54; +x_15 = x_55; +x_16 = x_71; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -4078,7 +4078,7 @@ lean_object* x_74; lean_object* x_75; lean_dec_ref(x_71); lean_dec_ref(x_69); lean_dec(x_68); -lean_dec_ref(x_53); +lean_dec_ref(x_55); lean_dec_ref(x_7); x_74 = lean_box(0); x_75 = lean_alloc_ctor(0, 1, 0); @@ -4089,11 +4089,11 @@ else { x_10 = x_68; x_11 = x_51; -x_12 = x_71; -x_13 = x_54; -x_14 = x_53; -x_15 = x_69; -x_16 = x_72; +x_12 = x_69; +x_13 = x_72; +x_14 = x_54; +x_15 = x_55; +x_16 = x_71; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -4105,18 +4105,18 @@ goto block_49; block_87: { lean_object* x_85; -x_85 = l_Lean_Syntax_getTailPos_x3f(x_78, x_81); -lean_dec(x_78); +x_85 = l_Lean_Syntax_getTailPos_x3f(x_83, x_79); +lean_dec(x_83); if (lean_obj_tag(x_85) == 0) { lean_inc(x_84); x_50 = x_77; x_51 = x_79; -x_52 = x_80; -x_53 = x_82; +x_52 = x_78; +x_53 = x_80; x_54 = x_81; -x_55 = x_84; -x_56 = x_83; +x_55 = x_82; +x_56 = x_84; x_57 = x_84; goto block_76; } @@ -4128,11 +4128,11 @@ lean_inc(x_86); lean_dec_ref(x_85); x_50 = x_77; x_51 = x_79; -x_52 = x_80; -x_53 = x_82; +x_52 = x_78; +x_53 = x_80; x_54 = x_81; -x_55 = x_84; -x_56 = x_83; +x_55 = x_82; +x_56 = x_84; x_57 = x_86; goto block_76; } @@ -4142,18 +4142,18 @@ goto block_76; lean_object* x_95; lean_object* x_96; x_95 = l_Lean_replaceRef(x_1, x_92); lean_dec(x_92); -x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_91); +x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_89); if (lean_obj_tag(x_96) == 0) { lean_object* x_97; x_97 = lean_unsigned_to_nat(0u); x_77 = x_88; -x_78 = x_95; -x_79 = x_94; -x_80 = x_89; -x_81 = x_91; -x_82 = x_90; -x_83 = x_93; +x_78 = x_90; +x_79 = x_89; +x_80 = x_91; +x_81 = x_94; +x_82 = x_93; +x_83 = x_95; x_84 = x_97; goto block_87; } @@ -4164,12 +4164,12 @@ x_98 = lean_ctor_get(x_96, 0); lean_inc(x_98); lean_dec_ref(x_96); x_77 = x_88; -x_78 = x_95; -x_79 = x_94; -x_80 = x_89; -x_81 = x_91; -x_82 = x_90; -x_83 = x_93; +x_78 = x_90; +x_79 = x_89; +x_80 = x_91; +x_81 = x_94; +x_82 = x_93; +x_83 = x_95; x_84 = x_98; goto block_87; } @@ -4178,23 +4178,23 @@ goto block_87; { if (x_107 == 0) { -x_88 = x_101; -x_89 = x_102; -x_90 = x_104; -x_91 = x_106; +x_88 = x_105; +x_89 = x_106; +x_90 = x_101; +x_91 = x_102; x_92 = x_103; -x_93 = x_105; +x_93 = x_104; x_94 = x_3; goto block_99; } else { -x_88 = x_101; -x_89 = x_102; -x_90 = x_104; -x_91 = x_106; +x_88 = x_105; +x_89 = x_106; +x_90 = x_101; +x_91 = x_102; x_92 = x_103; -x_93 = x_105; +x_93 = x_104; x_94 = x_100; goto block_99; } @@ -4218,14 +4218,14 @@ x_118 = 1; x_119 = l_Lean_instBEqMessageSeverity_beq(x_3, x_118); if (x_119 == 0) { -lean_inc_ref(x_111); lean_inc_ref(x_110); lean_inc(x_113); -x_101 = x_117; +lean_inc_ref(x_111); +x_101 = x_111; x_102 = x_114; x_103 = x_113; x_104 = x_110; -x_105 = x_111; +x_105 = x_117; x_106 = x_109; x_107 = x_119; goto block_108; @@ -4235,14 +4235,14 @@ else lean_object* x_120; uint8_t x_121; x_120 = l_Lean_logAt___at___00Lean_versoDocStringFromString_spec__3___redArg___closed__0; x_121 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_throwErrorAt___at___00Lean_parseVersoDocString___at___00Lean_versoDocString_spec__0_spec__1_spec__2_spec__5_spec__6(x_112, x_120); -lean_inc_ref(x_111); lean_inc_ref(x_110); lean_inc(x_113); -x_101 = x_117; +lean_inc_ref(x_111); +x_101 = x_111; x_102 = x_114; x_103 = x_113; x_104 = x_110; -x_105 = x_111; +x_105 = x_117; x_106 = x_109; x_107 = x_121; goto block_108; diff --git a/stage0/stdlib/Lean/DocString/Types.c b/stage0/stdlib/Lean/DocString/Types.c index e5c1b8efcea3..df79aff73ae7 100644 --- a/stage0/stdlib/Lean/DocString/Types.c +++ b/stage0/stdlib/Lean/DocString/Types.c @@ -6693,17 +6693,17 @@ if (lean_is_scalar(x_54)) { x_59 = x_54; lean_ctor_set_tag(x_59, 5); } -lean_ctor_set(x_59, 0, x_56); +lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); x_60 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_55); +lean_ctor_set(x_60, 1, x_56); x_61 = l_Array_Array_repr___redArg(x_7, x_53); x_62 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_62, 0, x_60); lean_ctor_set(x_62, 1, x_61); x_63 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_63, 0, x_57); +lean_ctor_set(x_63, 0, x_55); lean_ctor_set(x_63, 1, x_62); x_64 = 0; x_65 = lean_alloc_ctor(6, 1, 1); @@ -6726,9 +6726,9 @@ x_73 = l_Int_repr(x_52); lean_dec(x_52); x_74 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_74, 0, x_73); -x_55 = x_69; -x_56 = x_70; -x_57 = x_68; +x_55 = x_68; +x_56 = x_69; +x_57 = x_70; x_58 = x_74; goto block_67; } @@ -6741,9 +6741,9 @@ lean_dec(x_52); x_77 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_77, 0, x_76); x_78 = l_Repr_addAppParen(x_77, x_75); -x_55 = x_69; -x_56 = x_70; -x_57 = x_68; +x_55 = x_68; +x_56 = x_69; +x_57 = x_70; x_58 = x_78; goto block_67; } diff --git a/stage0/stdlib/Lean/Elab/Do/Legacy.c b/stage0/stdlib/Lean/Elab/Do/Legacy.c index 020fe5e9c421..a30fa1b5248f 100644 --- a/stage0/stdlib/Lean/Elab/Do/Legacy.c +++ b/stage0/stdlib/Lean/Elab/Do/Legacy.c @@ -8233,9 +8233,9 @@ goto block_115; block_108: { lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_nat_add(x_103, x_104); +x_105 = lean_nat_add(x_102, x_104); lean_dec(x_104); -lean_dec(x_103); +lean_dec(x_102); x_106 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_106, 0, x_105); lean_ctor_set(x_106, 1, x_81); @@ -8246,7 +8246,7 @@ x_107 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_107, 0, x_101); lean_ctor_set(x_107, 1, x_92); lean_ctor_set(x_107, 2, x_93); -lean_ctor_set(x_107, 3, x_102); +lean_ctor_set(x_107, 3, x_103); lean_ctor_set(x_107, 4, x_106); return x_107; } @@ -8268,8 +8268,8 @@ if (lean_obj_tag(x_95) == 0) lean_object* x_113; x_113 = lean_ctor_get(x_95, 0); lean_inc(x_113); -x_102 = x_111; -x_103 = x_112; +x_102 = x_112; +x_103 = x_111; x_104 = x_113; goto block_108; } @@ -8277,8 +8277,8 @@ else { lean_object* x_114; x_114 = lean_unsigned_to_nat(0u); -x_102 = x_111; -x_103 = x_112; +x_102 = x_112; +x_103 = x_111; x_104 = x_114; goto block_108; } @@ -9225,9 +9225,9 @@ goto block_204; block_196: { lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_193 = lean_nat_add(x_190, x_192); +x_193 = lean_nat_add(x_191, x_192); lean_dec(x_192); -lean_dec(x_190); +lean_dec(x_191); x_194 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_194, 0, x_193); lean_ctor_set(x_194, 1, x_170); @@ -9238,7 +9238,7 @@ x_195 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_195, 0, x_189); lean_ctor_set(x_195, 1, x_181); lean_ctor_set(x_195, 2, x_182); -lean_ctor_set(x_195, 3, x_191); +lean_ctor_set(x_195, 3, x_190); lean_ctor_set(x_195, 4, x_194); return x_195; } @@ -9260,8 +9260,8 @@ if (lean_obj_tag(x_184) == 0) lean_object* x_202; x_202 = lean_ctor_get(x_184, 0); lean_inc(x_202); -x_190 = x_201; -x_191 = x_200; +x_190 = x_200; +x_191 = x_201; x_192 = x_202; goto block_196; } @@ -9269,8 +9269,8 @@ else { lean_object* x_203; x_203 = lean_unsigned_to_nat(0u); -x_190 = x_201; -x_191 = x_200; +x_190 = x_200; +x_191 = x_201; x_192 = x_203; goto block_196; } @@ -9520,9 +9520,9 @@ goto block_276; block_268: { lean_object* x_265; lean_object* x_266; lean_object* x_267; -x_265 = lean_nat_add(x_262, x_264); +x_265 = lean_nat_add(x_263, x_264); lean_dec(x_264); -lean_dec(x_262); +lean_dec(x_263); x_266 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_266, 0, x_265); lean_ctor_set(x_266, 1, x_3); @@ -9533,7 +9533,7 @@ x_267 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_267, 0, x_261); lean_ctor_set(x_267, 1, x_253); lean_ctor_set(x_267, 2, x_254); -lean_ctor_set(x_267, 3, x_263); +lean_ctor_set(x_267, 3, x_262); lean_ctor_set(x_267, 4, x_266); return x_267; } @@ -9556,8 +9556,8 @@ if (lean_obj_tag(x_256) == 0) lean_object* x_274; x_274 = lean_ctor_get(x_256, 0); lean_inc(x_274); -x_262 = x_273; -x_263 = x_272; +x_262 = x_272; +x_263 = x_273; x_264 = x_274; goto block_268; } @@ -9565,8 +9565,8 @@ else { lean_object* x_275; x_275 = lean_unsigned_to_nat(0u); -x_262 = x_273; -x_263 = x_272; +x_262 = x_272; +x_263 = x_273; x_264 = x_275; goto block_268; } @@ -20887,8 +20887,8 @@ goto block_96; block_57: { 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_dec(x_37); lean_dec(x_36); +lean_dec(x_35); x_40 = l_Array_reverse___redArg(x_34); x_41 = lean_array_push(x_40, x_17); x_42 = l_Array_reverse___redArg(x_33); @@ -20901,8 +20901,8 @@ x_46 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_46, 0, x_39); lean_ctor_set(x_46, 1, x_45); x_47 = lean_array_size(x_44); -x_48 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Do_Legacy_0__Lean_Elab_Term_Do_expandDoIf_x3f_spec__3___redArg(x_19, x_8, x_9, x_10, x_11, x_16, x_30, x_44, x_47, x_25, x_46, x_35, x_38); -lean_dec_ref(x_35); +x_48 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Do_Legacy_0__Lean_Elab_Term_Do_expandDoIf_x3f_spec__3___redArg(x_19, x_8, x_9, x_10, x_11, x_16, x_30, x_44, x_47, x_25, x_46, x_38, x_37); +lean_dec_ref(x_38); lean_dec_ref(x_44); if (lean_obj_tag(x_48) == 0) { @@ -21016,10 +21016,10 @@ x_92 = l_Lean_Syntax_node2(x_71, x_74, x_89, x_91); lean_inc(x_71); x_93 = l_Lean_Syntax_node1(x_71, x_73, x_92); x_94 = l_Lean_Syntax_node1(x_71, x_72, x_93); -x_35 = x_68; -x_36 = x_69; -x_37 = x_70; -x_38 = x_60; +x_35 = x_69; +x_36 = x_70; +x_37 = x_60; +x_38 = x_68; x_39 = x_94; goto block_57; } @@ -21032,10 +21032,10 @@ lean_dec(x_62); x_95 = lean_ctor_get(x_58, 0); lean_inc(x_95); lean_dec_ref(x_58); -x_35 = x_68; -x_36 = x_69; -x_37 = x_70; -x_38 = x_60; +x_35 = x_69; +x_36 = x_70; +x_37 = x_60; +x_38 = x_68; x_39 = x_95; goto block_57; } @@ -21226,11 +21226,11 @@ return x_211; block_134: { 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; size_t x_123; size_t x_124; lean_object* x_125; -lean_dec(x_113); -lean_dec(x_109); -x_116 = l_Array_reverse___redArg(x_114); +lean_dec(x_114); +lean_dec(x_110); +x_116 = l_Array_reverse___redArg(x_109); x_117 = lean_array_push(x_116, x_17); -x_118 = l_Array_reverse___redArg(x_112); +x_118 = l_Array_reverse___redArg(x_111); x_119 = lean_array_push(x_118, x_108); x_120 = l_Array_zip___redArg(x_117, x_119); lean_dec_ref(x_119); @@ -21241,8 +21241,8 @@ lean_ctor_set(x_122, 0, x_115); lean_ctor_set(x_122, 1, x_121); x_123 = lean_array_size(x_120); x_124 = 0; -x_125 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Do_Legacy_0__Lean_Elab_Term_Do_expandDoIf_x3f_spec__4___redArg(x_8, x_9, x_10, x_11, x_16, x_106, x_120, x_123, x_124, x_122, x_110, x_111); -lean_dec_ref(x_110); +x_125 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Do_Legacy_0__Lean_Elab_Term_Do_expandDoIf_x3f_spec__4___redArg(x_8, x_9, x_10, x_11, x_16, x_106, x_120, x_123, x_124, x_122, x_112, x_113); +lean_dec_ref(x_112); lean_dec_ref(x_120); if (lean_obj_tag(x_125) == 0) { @@ -21357,12 +21357,12 @@ x_172 = l_Lean_Syntax_node2(x_151, x_154, x_169, x_171); lean_inc(x_151); x_173 = l_Lean_Syntax_node1(x_151, x_153, x_172); x_174 = l_Lean_Syntax_node1(x_151, x_152, x_173); -x_109 = x_149; -x_110 = x_147; -x_111 = x_139; -x_112 = x_136; -x_113 = x_148; -x_114 = x_135; +x_109 = x_135; +x_110 = x_149; +x_111 = x_136; +x_112 = x_147; +x_113 = x_139; +x_114 = x_148; x_115 = x_174; goto block_134; } @@ -21375,12 +21375,12 @@ lean_dec(x_141); x_175 = lean_ctor_get(x_137, 0); lean_inc(x_175); lean_dec_ref(x_137); -x_109 = x_149; -x_110 = x_147; -x_111 = x_139; -x_112 = x_136; -x_113 = x_148; -x_114 = x_135; +x_109 = x_135; +x_110 = x_149; +x_111 = x_136; +x_112 = x_147; +x_113 = x_139; +x_114 = x_148; x_115 = x_175; goto block_134; } @@ -39515,7 +39515,7 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Do_ToCodeBlock_doTryToCode(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_11; uint8_t x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +uint8_t x_11; lean_object* x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; x_51 = lean_unsigned_to_nat(1u); x_52 = l_Lean_Syntax_getArg(x_1, x_51); x_53 = l___private_Lean_Elab_Do_Legacy_0__Lean_Elab_Term_getDoSeqElems(x_52); @@ -39549,7 +39549,7 @@ lean_inc_ref(x_3); x_61 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Elab_Term_Do_ToCodeBlock_doTryToCode_spec__2(x_51, x_59, x_60, x_58, x_3, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_61) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; lean_object* x_77; uint8_t x_78; lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; 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_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; 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; uint8_t x_195; +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; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; uint8_t x_76; lean_object* x_77; uint8_t x_78; lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; uint8_t x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; 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_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; 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; uint8_t x_195; x_62 = lean_ctor_get(x_61, 0); lean_inc(x_62); lean_dec_ref(x_61); @@ -39626,22 +39626,22 @@ goto block_194; block_105: { 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_object* x_92; uint8_t x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_79 = lean_ctor_get(x_74, 0); -x_80 = lean_ctor_get(x_74, 1); -x_81 = lean_ctor_get(x_74, 2); -x_82 = lean_ctor_get(x_74, 3); -x_83 = lean_ctor_get(x_74, 4); -x_84 = lean_ctor_get(x_74, 5); -x_85 = lean_ctor_get(x_74, 6); -x_86 = lean_ctor_get(x_74, 7); -x_87 = lean_ctor_get(x_74, 8); -x_88 = lean_ctor_get(x_74, 9); -x_89 = lean_ctor_get(x_74, 10); -x_90 = lean_ctor_get(x_74, 11); -x_91 = lean_ctor_get_uint8(x_74, sizeof(void*)*14); -x_92 = lean_ctor_get(x_74, 12); -x_93 = lean_ctor_get_uint8(x_74, sizeof(void*)*14 + 1); -x_94 = lean_ctor_get(x_74, 13); +x_79 = lean_ctor_get(x_71, 0); +x_80 = lean_ctor_get(x_71, 1); +x_81 = lean_ctor_get(x_71, 2); +x_82 = lean_ctor_get(x_71, 3); +x_83 = lean_ctor_get(x_71, 4); +x_84 = lean_ctor_get(x_71, 5); +x_85 = lean_ctor_get(x_71, 6); +x_86 = lean_ctor_get(x_71, 7); +x_87 = lean_ctor_get(x_71, 8); +x_88 = lean_ctor_get(x_71, 9); +x_89 = lean_ctor_get(x_71, 10); +x_90 = lean_ctor_get(x_71, 11); +x_91 = lean_ctor_get_uint8(x_71, sizeof(void*)*14); +x_92 = lean_ctor_get(x_71, 12); +x_93 = lean_ctor_get_uint8(x_71, sizeof(void*)*14 + 1); +x_94 = lean_ctor_get(x_71, 13); x_95 = l_Lean_replaceRef(x_64, x_84); lean_dec(x_64); lean_inc_ref(x_94); @@ -39678,31 +39678,31 @@ if (x_78 == 0) { lean_object* x_97; lean_object* x_98; x_97 = l_Lean_Elab_Term_Do_ToCodeBlock_doTryToCode___closed__1; -x_98 = l_Lean_throwError___at___00Lean_Elab_Term_Do_ToCodeBlock_checkReassignable_spec__0___redArg(x_97, x_72, x_65, x_96, x_68); +x_98 = l_Lean_throwError___at___00Lean_Elab_Term_Do_ToCodeBlock_checkReassignable_spec__0___redArg(x_97, x_73, x_72, x_96, x_65); if (lean_obj_tag(x_98) == 0) { lean_object* x_99; lean_object* x_100; x_99 = lean_ctor_get(x_98, 0); lean_inc(x_99); lean_dec_ref(x_98); -lean_inc(x_68); lean_inc(x_65); -lean_inc_ref(x_72); -lean_inc(x_73); +lean_inc(x_72); +lean_inc_ref(x_73); +lean_inc(x_68); +lean_inc_ref(x_70); lean_inc_ref(x_75); -lean_inc_ref(x_69); -x_100 = lean_apply_9(x_71, x_99, x_69, x_75, x_73, x_72, x_65, x_96, x_68, lean_box(0)); +x_100 = lean_apply_9(x_66, x_99, x_75, x_70, x_68, x_73, x_72, x_96, x_65, lean_box(0)); x_35 = x_65; -x_36 = x_70; -x_37 = x_72; -x_38 = x_73; -x_39 = x_66; -x_40 = x_74; -x_41 = x_76; -x_42 = x_75; +x_36 = x_69; +x_37 = x_70; +x_38 = x_71; +x_39 = x_72; +x_40 = x_67; +x_41 = x_74; +x_42 = x_73; x_43 = x_68; -x_44 = x_69; -x_45 = x_77; +x_44 = x_75; +x_45 = x_76; x_46 = x_100; goto block_50; } @@ -39710,14 +39710,14 @@ else { lean_object* x_101; lean_object* x_102; lean_dec_ref(x_96); -lean_dec_ref(x_77); lean_dec_ref(x_75); -lean_dec_ref(x_74); -lean_dec(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_73); +lean_dec(x_72); lean_dec_ref(x_71); -lean_dec_ref(x_69); +lean_dec_ref(x_70); lean_dec(x_68); +lean_dec_ref(x_67); +lean_dec_ref(x_66); lean_dec(x_65); lean_dec(x_2); x_101 = lean_ctor_get(x_98, 0); @@ -39732,57 +39732,57 @@ else { lean_object* x_103; lean_object* x_104; x_103 = lean_box(0); -lean_inc(x_68); lean_inc(x_65); -lean_inc_ref(x_72); -lean_inc(x_73); +lean_inc(x_72); +lean_inc_ref(x_73); +lean_inc(x_68); +lean_inc_ref(x_70); lean_inc_ref(x_75); -lean_inc_ref(x_69); -x_104 = lean_apply_9(x_71, x_103, x_69, x_75, x_73, x_72, x_65, x_96, x_68, lean_box(0)); +x_104 = lean_apply_9(x_66, x_103, x_75, x_70, x_68, x_73, x_72, x_96, x_65, lean_box(0)); x_35 = x_65; -x_36 = x_70; -x_37 = x_72; -x_38 = x_73; -x_39 = x_66; -x_40 = x_74; -x_41 = x_76; -x_42 = x_75; +x_36 = x_69; +x_37 = x_70; +x_38 = x_71; +x_39 = x_72; +x_40 = x_67; +x_41 = x_74; +x_42 = x_73; x_43 = x_68; -x_44 = x_69; -x_45 = x_77; +x_44 = x_75; +x_45 = x_76; x_46 = x_104; goto block_50; } } block_128: { -if (lean_obj_tag(x_116) == 0) +if (lean_obj_tag(x_119) == 0) { lean_dec(x_107); lean_dec(x_106); lean_dec(x_64); lean_dec(x_1); x_11 = x_109; -x_12 = x_112; +x_12 = x_113; x_13 = x_114; -x_14 = x_119; +x_14 = x_118; x_15 = x_120; -x_16 = x_118; -x_17 = x_115; -x_18 = x_111; -x_19 = x_110; -x_20 = x_108; -x_21 = x_113; -x_22 = x_117; +x_16 = x_117; +x_17 = x_110; +x_18 = x_116; +x_19 = x_115; +x_20 = x_112; +x_21 = x_111; +x_22 = x_108; x_23 = lean_box(0); goto block_34; } else { lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_122 = lean_ctor_get(x_116, 0); +x_122 = lean_ctor_get(x_119, 0); lean_inc(x_122); -lean_dec_ref(x_116); +lean_dec_ref(x_119); x_123 = lean_ctor_get(x_122, 0); lean_inc_ref(x_123); x_124 = lean_ctor_get(x_122, 1); @@ -39800,18 +39800,18 @@ uint8_t x_126; lean_dec_ref(x_124); x_126 = 0; x_65 = x_108; -x_66 = x_112; -x_67 = lean_box(0); -x_68 = x_117; -x_69 = x_118; -x_70 = x_109; -x_71 = x_125; -x_72 = x_110; -x_73 = x_111; -x_74 = x_113; -x_75 = x_115; -x_76 = x_114; -x_77 = x_119; +x_66 = x_125; +x_67 = x_113; +x_68 = x_116; +x_69 = x_109; +x_70 = x_110; +x_71 = x_111; +x_72 = x_112; +x_73 = x_115; +x_74 = x_114; +x_75 = x_117; +x_76 = x_118; +x_77 = lean_box(0); x_78 = x_126; goto block_105; } @@ -39820,18 +39820,18 @@ else uint8_t x_127; x_127 = 1; x_65 = x_108; -x_66 = x_112; -x_67 = lean_box(0); -x_68 = x_117; -x_69 = x_118; -x_70 = x_109; -x_71 = x_125; -x_72 = x_110; -x_73 = x_111; -x_74 = x_113; -x_75 = x_115; -x_76 = x_114; -x_77 = x_119; +x_66 = x_125; +x_67 = x_113; +x_68 = x_116; +x_69 = x_109; +x_70 = x_110; +x_71 = x_111; +x_72 = x_112; +x_73 = x_115; +x_74 = x_114; +x_75 = x_117; +x_76 = x_118; +x_77 = lean_box(0); x_78 = x_127; goto block_105; } @@ -39909,18 +39909,18 @@ lean_dec(x_138); lean_dec(x_62); x_106 = x_143; x_107 = x_142; -x_108 = x_134; -x_109 = x_146; -x_110 = x_133; -x_111 = x_132; -x_112 = x_150; -x_113 = x_135; -x_114 = x_148; -x_115 = x_131; -x_116 = x_129; -x_117 = x_136; -x_118 = x_130; -x_119 = x_144; +x_108 = x_136; +x_109 = x_148; +x_110 = x_131; +x_111 = x_135; +x_112 = x_134; +x_113 = x_144; +x_114 = x_150; +x_115 = x_133; +x_116 = x_132; +x_117 = x_130; +x_118 = x_146; +x_119 = x_129; x_120 = x_156; x_121 = lean_box(0); goto block_128; @@ -39935,18 +39935,18 @@ lean_dec(x_138); lean_dec(x_62); x_106 = x_143; x_107 = x_142; -x_108 = x_134; -x_109 = x_146; -x_110 = x_133; -x_111 = x_132; -x_112 = x_150; -x_113 = x_135; -x_114 = x_148; -x_115 = x_131; -x_116 = x_129; -x_117 = x_136; -x_118 = x_130; -x_119 = x_144; +x_108 = x_136; +x_109 = x_148; +x_110 = x_131; +x_111 = x_135; +x_112 = x_134; +x_113 = x_144; +x_114 = x_150; +x_115 = x_133; +x_116 = x_132; +x_117 = x_130; +x_118 = x_146; +x_119 = x_129; x_120 = x_156; x_121 = lean_box(0); goto block_128; @@ -39974,18 +39974,18 @@ lean_inc(x_163); lean_dec_ref(x_162); x_106 = x_143; x_107 = x_142; -x_108 = x_134; -x_109 = x_146; -x_110 = x_133; -x_111 = x_132; -x_112 = x_150; -x_113 = x_135; -x_114 = x_148; -x_115 = x_131; -x_116 = x_129; -x_117 = x_136; -x_118 = x_130; -x_119 = x_144; +x_108 = x_136; +x_109 = x_148; +x_110 = x_131; +x_111 = x_135; +x_112 = x_134; +x_113 = x_144; +x_114 = x_150; +x_115 = x_133; +x_116 = x_132; +x_117 = x_130; +x_118 = x_146; +x_119 = x_129; x_120 = x_163; x_121 = lean_box(0); goto block_128; @@ -40067,14 +40067,14 @@ return x_139; { if (x_178 == 0) { -x_129 = x_172; -x_130 = x_170; -x_131 = x_169; -x_132 = x_177; -x_133 = x_175; -x_134 = x_171; -x_135 = x_174; -x_136 = x_176; +x_129 = x_176; +x_130 = x_171; +x_131 = x_173; +x_132 = x_170; +x_133 = x_169; +x_134 = x_177; +x_135 = x_175; +x_136 = x_172; x_137 = lean_box(0); goto block_168; } @@ -40082,18 +40082,18 @@ else { lean_object* x_179; lean_object* x_180; x_179 = l_Lean_Elab_Term_Do_ToCodeBlock_doTryToCode___closed__6; -x_180 = l_Lean_throwError___at___00Lean_Elab_Term_Do_ToCodeBlock_checkReassignable_spec__0___redArg(x_179, x_175, x_171, x_174, x_176); +x_180 = l_Lean_throwError___at___00Lean_Elab_Term_Do_ToCodeBlock_checkReassignable_spec__0___redArg(x_179, x_169, x_177, x_175, x_172); if (lean_obj_tag(x_180) == 0) { lean_dec_ref(x_180); -x_129 = x_172; -x_130 = x_170; -x_131 = x_169; -x_132 = x_177; -x_133 = x_175; -x_134 = x_171; -x_135 = x_174; -x_136 = x_176; +x_129 = x_176; +x_130 = x_171; +x_131 = x_173; +x_132 = x_170; +x_133 = x_169; +x_134 = x_177; +x_135 = x_175; +x_136 = x_172; x_137 = lean_box(0); goto block_168; } @@ -40103,10 +40103,10 @@ lean_object* x_181; lean_object* x_182; lean_dec(x_177); lean_dec(x_176); lean_dec_ref(x_175); -lean_dec_ref(x_174); +lean_dec_ref(x_173); lean_dec(x_172); -lean_dec(x_171); -lean_dec_ref(x_170); +lean_dec_ref(x_171); +lean_dec(x_170); lean_dec_ref(x_169); lean_dec(x_64); lean_dec(x_62); @@ -40128,15 +40128,15 @@ uint8_t x_193; x_193 = l_Array_isEmpty___redArg(x_62); if (x_193 == 0) { -x_169 = x_186; -x_170 = x_185; -x_171 = x_189; -x_172 = x_184; -x_173 = lean_box(0); -x_174 = x_190; -x_175 = x_188; -x_176 = x_191; -x_177 = x_187; +x_169 = x_188; +x_170 = x_187; +x_171 = x_185; +x_172 = x_191; +x_173 = x_186; +x_174 = lean_box(0); +x_175 = x_190; +x_176 = x_184; +x_177 = x_189; x_178 = x_193; goto block_183; } @@ -40144,15 +40144,15 @@ else { if (lean_obj_tag(x_184) == 0) { -x_169 = x_186; -x_170 = x_185; -x_171 = x_189; -x_172 = x_184; -x_173 = lean_box(0); -x_174 = x_190; -x_175 = x_188; -x_176 = x_191; -x_177 = x_187; +x_169 = x_188; +x_170 = x_187; +x_171 = x_185; +x_172 = x_191; +x_173 = x_186; +x_174 = lean_box(0); +x_175 = x_190; +x_176 = x_184; +x_177 = x_189; x_178 = x_193; goto block_183; } @@ -40209,12 +40209,12 @@ return x_54; block_34: { lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_box(x_11); -x_25 = lean_box(x_13); -x_26 = lean_box(x_12); +x_24 = lean_box(x_14); +x_25 = lean_box(x_11); +x_26 = lean_box(x_13); x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Do_ToTerm_matchNestedTermResult___boxed), 7, 5); lean_closure_set(x_27, 0, x_15); -lean_closure_set(x_27, 1, x_14); +lean_closure_set(x_27, 1, x_12); lean_closure_set(x_27, 2, x_24); lean_closure_set(x_27, 3, x_25); lean_closure_set(x_27, 4, x_26); @@ -40258,29 +40258,29 @@ x_47 = lean_ctor_get(x_46, 0); lean_inc(x_47); lean_dec_ref(x_46); x_11 = x_36; -x_12 = x_39; +x_12 = x_40; x_13 = x_41; x_14 = x_45; x_15 = x_47; x_16 = x_44; -x_17 = x_42; -x_18 = x_38; -x_19 = x_37; -x_20 = x_35; -x_21 = x_40; -x_22 = x_43; +x_17 = x_37; +x_18 = x_43; +x_19 = x_42; +x_20 = x_39; +x_21 = x_38; +x_22 = x_35; x_23 = lean_box(0); goto block_34; } else { lean_object* x_48; lean_object* x_49; -lean_dec_ref(x_45); lean_dec_ref(x_44); lean_dec(x_43); lean_dec_ref(x_42); lean_dec_ref(x_40); -lean_dec(x_38); +lean_dec(x_39); +lean_dec_ref(x_38); lean_dec_ref(x_37); lean_dec(x_35); lean_dec(x_2); diff --git a/stage0/stdlib/Lean/Elab/DocString.c b/stage0/stdlib/Lean/Elab/DocString.c index 2d206ccc9129..ecd12d318fa6 100644 --- a/stage0/stdlib/Lean/Elab/DocString.c +++ b/stage0/stdlib/Lean/Elab/DocString.c @@ -43587,8 +43587,8 @@ if (lean_obj_tag(x_49) == 0) { lean_object* x_50; x_50 = l_Std_DTreeMap_Internal_Impl_Const_alter___at___00Lean_Doc_addBuiltinDocRole_spec__0___redArg___lam__0___closed__0; -x_30 = lean_box(0); -x_31 = x_46; +x_30 = x_46; +x_31 = lean_box(0); x_32 = x_50; goto block_42; } @@ -43598,8 +43598,8 @@ lean_object* x_51; x_51 = lean_ctor_get(x_49, 0); lean_inc(x_51); lean_dec_ref(x_49); -x_30 = lean_box(0); -x_31 = x_46; +x_30 = x_46; +x_31 = lean_box(0); x_32 = x_51; goto block_42; } @@ -43749,9 +43749,9 @@ goto block_22; block_42: { size_t x_33; size_t x_34; lean_object* x_35; -x_33 = lean_array_size(x_31); +x_33 = lean_array_size(x_30); x_34 = 0; -x_35 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_DocString_0__Lean_Doc_roleExpandersForUnsafe_spec__0(x_33, x_34, x_31, x_2, x_3, x_4, x_5, x_6, x_7); +x_35 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_DocString_0__Lean_Doc_roleExpandersForUnsafe_spec__0(x_33, x_34, x_30, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_7); lean_dec_ref(x_6); if (lean_obj_tag(x_35) == 0) @@ -44437,8 +44437,8 @@ if (lean_obj_tag(x_49) == 0) { lean_object* x_50; x_50 = l_Std_DTreeMap_Internal_Impl_Const_alter___at___00Lean_Doc_addBuiltinDocDirective_spec__0___redArg___lam__0___closed__0; -x_30 = x_46; -x_31 = lean_box(0); +x_30 = lean_box(0); +x_31 = x_46; x_32 = x_50; goto block_42; } @@ -44448,8 +44448,8 @@ lean_object* x_51; x_51 = lean_ctor_get(x_49, 0); lean_inc(x_51); lean_dec_ref(x_49); -x_30 = x_46; -x_31 = lean_box(0); +x_30 = lean_box(0); +x_31 = x_46; x_32 = x_51; goto block_42; } @@ -44599,9 +44599,9 @@ goto block_22; block_42: { size_t x_33; size_t x_34; lean_object* x_35; -x_33 = lean_array_size(x_30); +x_33 = lean_array_size(x_31); x_34 = 0; -x_35 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_DocString_0__Lean_Doc_directiveExpandersForUnsafe_spec__0(x_33, x_34, x_30, x_2, x_3, x_4, x_5, x_6, x_7); +x_35 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_DocString_0__Lean_Doc_directiveExpandersForUnsafe_spec__0(x_33, x_34, x_31, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_7); lean_dec_ref(x_6); if (lean_obj_tag(x_35) == 0) @@ -45499,7 +45499,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_logWarningAt___at___00__private_Lean_Elab_DocString_0__Lean_Doc_mkArg_spec__0_spec__0___redArg(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) { _start: { -lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_47; uint8_t x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_56; uint8_t x_57; uint8_t x_58; lean_object* x_59; uint8_t x_60; lean_object* x_71; uint8_t x_72; uint8_t x_73; lean_object* x_74; uint8_t x_75; uint8_t x_76; uint8_t x_78; uint8_t x_91; +lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_56; uint8_t x_57; uint8_t x_58; lean_object* x_59; uint8_t x_60; lean_object* x_71; uint8_t x_72; uint8_t x_73; lean_object* x_74; uint8_t x_75; uint8_t x_76; uint8_t x_78; uint8_t x_91; x_13 = l_Lean_logAt___at___00Lean_logWarningAt___at___00__private_Lean_Elab_DocString_0__Lean_Doc_mkArg_spec__0_spec__0___redArg___closed__0; x_14 = l_Lean_logAt___at___00Lean_logWarningAt___at___00__private_Lean_Elab_DocString_0__Lean_Doc_mkArg_spec__0_spec__0___redArg___closed__1; x_56 = l_Lean_logAt___at___00Lean_logWarningAt___at___00__private_Lean_Elab_DocString_0__Lean_Doc_mkArg_spec__0_spec__0___redArg___closed__2; @@ -45565,15 +45565,15 @@ x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); lean_dec_ref(x_26); lean_inc(x_21); -x_28 = l_Lean_FileMap_toPosition(x_21, x_18); -lean_dec(x_18); +x_28 = l_Lean_FileMap_toPosition(x_21, x_17); +lean_dec(x_17); x_29 = l_Lean_FileMap_toPosition(x_21, x_19); lean_dec(x_19); x_30 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_30, 0, x_29); x_31 = l___private_Lean_Elab_DocString_0__Lean_Doc_getModState___redArg___lam__6___closed__1; -x_32 = lean_box(x_16); -x_33 = lean_box(x_15); +x_32 = lean_box(x_15); +x_33 = lean_box(x_16); x_34 = lean_box(x_4); x_35 = lean_alloc_closure((void*)(l_Lean_logAt___at___00Lean_logErrorAt___at___00Lean_Doc_done_spec__0_spec__0___redArg___lam__6___boxed), 15, 8); lean_closure_set(x_35, 0, x_25); @@ -45593,7 +45593,7 @@ uint8_t x_37; lean_dec(x_25); lean_dec(x_21); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_11); lean_dec_ref(x_10); lean_dec(x_9); @@ -45622,7 +45622,7 @@ else uint8_t x_40; lean_dec(x_21); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_11); lean_dec_ref(x_10); lean_dec(x_9); @@ -45650,7 +45650,7 @@ else { uint8_t x_43; lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_11); lean_dec_ref(x_10); lean_dec(x_9); @@ -45678,15 +45678,15 @@ return x_45; block_55: { lean_object* x_53; -x_53 = l_Lean_Syntax_getTailPos_x3f(x_51, x_50); -lean_dec(x_51); +x_53 = l_Lean_Syntax_getTailPos_x3f(x_50, x_51); +lean_dec(x_50); if (lean_obj_tag(x_53) == 0) { lean_inc(x_52); x_15 = x_47; -x_16 = x_48; -x_17 = lean_box(0); -x_18 = x_52; +x_16 = x_49; +x_17 = x_52; +x_18 = lean_box(0); x_19 = x_52; goto block_46; } @@ -45697,9 +45697,9 @@ x_54 = lean_ctor_get(x_53, 0); lean_inc(x_54); lean_dec_ref(x_53); x_15 = x_47; -x_16 = x_48; -x_17 = lean_box(0); -x_18 = x_52; +x_16 = x_49; +x_17 = x_52; +x_18 = lean_box(0); x_19 = x_54; goto block_46; } @@ -45727,11 +45727,11 @@ if (lean_obj_tag(x_64) == 0) { lean_object* x_65; x_65 = lean_unsigned_to_nat(0u); -x_47 = x_60; -x_48 = x_57; -x_49 = lean_box(0); -x_50 = x_58; -x_51 = x_63; +x_47 = x_57; +x_48 = lean_box(0); +x_49 = x_60; +x_50 = x_63; +x_51 = x_58; x_52 = x_65; goto block_55; } @@ -45741,11 +45741,11 @@ lean_object* x_66; x_66 = lean_ctor_get(x_64, 0); lean_inc(x_66); lean_dec_ref(x_64); -x_47 = x_60; -x_48 = x_57; -x_49 = lean_box(0); -x_50 = x_58; -x_51 = x_63; +x_47 = x_57; +x_48 = lean_box(0); +x_49 = x_60; +x_50 = x_63; +x_51 = x_58; x_52 = x_66; goto block_55; } @@ -53938,10 +53938,10 @@ goto block_37; { if (x_22 == 0) { -if (lean_obj_tag(x_21) == 1) +if (lean_obj_tag(x_20) == 1) { lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = lean_ctor_get(x_21, 0); +x_23 = lean_ctor_get(x_20, 0); x_24 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_elabInline_spec__2___closed__0; x_25 = l_Lean_instBEqInternalExceptionId_beq(x_23, x_24); if (x_25 == 0) @@ -53960,13 +53960,13 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_21); +lean_ctor_set(x_26, 0, x_20); return x_26; } else { size_t x_27; size_t x_28; -lean_dec_ref(x_21); +lean_dec_ref(x_20); x_27 = 1; x_28 = lean_usize_add(x_8, x_27); lean_inc_ref(x_1); @@ -53995,7 +53995,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_21); +lean_ctor_set(x_30, 0, x_20); return x_30; } } @@ -54015,7 +54015,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_31 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_31, 0, x_21); +lean_ctor_set(x_31, 0, x_20); return x_31; } } @@ -54028,15 +54028,15 @@ if (x_35 == 0) uint8_t x_36; lean_inc_ref(x_33); x_36 = l_Lean_Exception_isRuntime(x_33); -x_20 = lean_box(0); -x_21 = x_33; +x_20 = x_33; +x_21 = lean_box(0); x_22 = x_36; goto block_32; } else { -x_20 = lean_box(0); -x_21 = x_33; +x_20 = x_33; +x_21 = lean_box(0); x_22 = x_35; goto block_32; } @@ -58371,10 +58371,10 @@ goto block_37; { if (x_22 == 0) { -if (lean_obj_tag(x_20) == 1) +if (lean_obj_tag(x_21) == 1) { lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_21, 0); x_24 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_elabInline_spec__2___closed__0; x_25 = l_Lean_instBEqInternalExceptionId_beq(x_23, x_24); if (x_25 == 0) @@ -58393,13 +58393,13 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_20); +lean_ctor_set(x_26, 0, x_21); return x_26; } else { size_t x_27; size_t x_28; -lean_dec_ref(x_20); +lean_dec_ref(x_21); x_27 = 1; x_28 = lean_usize_add(x_8, x_27); lean_inc_ref(x_1); @@ -58428,7 +58428,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_20); +lean_ctor_set(x_30, 0, x_21); return x_30; } } @@ -58448,7 +58448,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_31 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_31, 0, x_20); +lean_ctor_set(x_31, 0, x_21); return x_31; } } @@ -58461,15 +58461,15 @@ if (x_35 == 0) uint8_t x_36; lean_inc_ref(x_33); x_36 = l_Lean_Exception_isRuntime(x_33); -x_20 = x_33; -x_21 = lean_box(0); +x_20 = lean_box(0); +x_21 = x_33; x_22 = x_36; goto block_32; } else { -x_20 = x_33; -x_21 = lean_box(0); +x_20 = lean_box(0); +x_21 = x_33; x_22 = x_35; goto block_32; } diff --git a/stage0/stdlib/Lean/Elab/DocString/Builtin.c b/stage0/stdlib/Lean/Elab/DocString/Builtin.c index c8be45707b6b..f02fa4e73161 100644 --- a/stage0/stdlib/Lean/Elab/DocString/Builtin.c +++ b/stage0/stdlib/Lean/Elab/DocString/Builtin.c @@ -44703,7 +44703,7 @@ return x_7; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_logInfoAt___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_lean_runCommand_spec__0_spec__0(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -uint8_t 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; uint8_t x_82; uint8_t x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; uint8_t x_116; lean_object* x_117; uint8_t x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; uint8_t x_125; uint8_t x_126; lean_object* x_127; uint8_t x_128; uint8_t x_139; uint8_t x_140; uint8_t x_141; lean_object* x_142; uint8_t x_143; uint8_t x_145; uint8_t x_158; +lean_object* x_8; uint8_t x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_82; uint8_t x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; uint8_t x_116; lean_object* x_117; uint8_t x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; uint8_t x_125; lean_object* x_126; uint8_t x_127; uint8_t x_128; uint8_t x_139; uint8_t x_140; lean_object* x_141; uint8_t x_142; uint8_t x_143; uint8_t x_145; uint8_t x_158; x_139 = 2; x_158 = l_Lean_instBEqMessageSeverity_beq(x_3, x_139); if (x_158 == 0) @@ -44755,15 +44755,15 @@ lean_ctor_set(x_27, 0, x_23); lean_ctor_set(x_27, 1, x_24); x_28 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_13); +lean_ctor_set(x_28, 1, x_8); x_29 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_29, 0, x_10); -lean_ctor_set(x_29, 1, x_14); -lean_ctor_set(x_29, 2, x_12); +lean_ctor_set(x_29, 0, x_12); +lean_ctor_set(x_29, 1, x_13); +lean_ctor_set(x_29, 2, x_14); lean_ctor_set(x_29, 3, x_11); lean_ctor_set(x_29, 4, x_28); lean_ctor_set_uint8(x_29, sizeof(void*)*5, x_9); -lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 1, x_8); +lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 1, x_10); lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 2, x_4); x_30 = l_Lean_MessageLog_add(x_29, x_26); lean_ctor_set(x_22, 1, x_30); @@ -44803,15 +44803,15 @@ lean_ctor_set(x_44, 0, x_23); lean_ctor_set(x_44, 1, x_24); x_45 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_13); +lean_ctor_set(x_45, 1, x_8); x_46 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_46, 0, x_10); -lean_ctor_set(x_46, 1, x_14); -lean_ctor_set(x_46, 2, x_12); +lean_ctor_set(x_46, 0, x_12); +lean_ctor_set(x_46, 1, x_13); +lean_ctor_set(x_46, 2, x_14); lean_ctor_set(x_46, 3, x_11); lean_ctor_set(x_46, 4, x_45); lean_ctor_set_uint8(x_46, sizeof(void*)*5, x_9); -lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 1, x_8); +lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 1, x_10); lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 2, x_4); x_47 = l_Lean_MessageLog_add(x_46, x_34); x_48 = lean_alloc_ctor(0, 11, 0); @@ -44889,15 +44889,15 @@ lean_ctor_set(x_67, 0, x_53); lean_ctor_set(x_67, 1, x_54); x_68 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_13); +lean_ctor_set(x_68, 1, x_8); x_69 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_69, 0, x_10); -lean_ctor_set(x_69, 1, x_14); -lean_ctor_set(x_69, 2, x_12); +lean_ctor_set(x_69, 0, x_12); +lean_ctor_set(x_69, 1, x_13); +lean_ctor_set(x_69, 2, x_14); lean_ctor_set(x_69, 3, x_11); lean_ctor_set(x_69, 4, x_68); lean_ctor_set_uint8(x_69, sizeof(void*)*5, x_9); -lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 1, x_8); +lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 1, x_10); lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 2, x_4); x_70 = l_Lean_MessageLog_add(x_69, x_56); if (lean_is_scalar(x_66)) { @@ -44927,11 +44927,11 @@ else { uint8_t x_75; lean_dec(x_18); -lean_dec_ref(x_14); +lean_dec(x_14); lean_dec_ref(x_13); -lean_dec(x_12); +lean_dec_ref(x_12); lean_dec_ref(x_11); -lean_dec_ref(x_10); +lean_dec_ref(x_8); x_75 = !lean_is_exclusive(x_19); if (x_75 == 0) { @@ -44952,11 +44952,11 @@ return x_77; else { uint8_t x_78; -lean_dec_ref(x_14); +lean_dec(x_14); lean_dec_ref(x_13); -lean_dec(x_12); +lean_dec_ref(x_12); lean_dec_ref(x_11); -lean_dec_ref(x_10); +lean_dec_ref(x_8); x_78 = !lean_is_exclusive(x_17); if (x_78 == 0) { @@ -45001,13 +45001,13 @@ x_98 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraM if (x_90 == 0) { lean_free_object(x_92); -x_8 = x_83; -x_9 = x_85; -x_10 = x_88; +x_8 = x_94; +x_9 = x_83; +x_10 = x_85; x_11 = x_98; -x_12 = x_97; -x_13 = x_94; -x_14 = x_95; +x_12 = x_88; +x_13 = x_95; +x_14 = x_97; x_15 = x_6; x_16 = lean_box(0); goto block_81; @@ -45036,13 +45036,13 @@ return x_92; else { lean_free_object(x_92); -x_8 = x_83; -x_9 = x_85; -x_10 = x_88; +x_8 = x_94; +x_9 = x_83; +x_10 = x_85; x_11 = x_98; -x_12 = x_97; -x_13 = x_94; -x_14 = x_95; +x_12 = x_88; +x_13 = x_95; +x_14 = x_97; x_15 = x_6; x_16 = lean_box(0); goto block_81; @@ -45065,13 +45065,13 @@ lean_ctor_set(x_107, 0, x_106); x_108 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_elabExtraTerm_spec__0_spec__0_spec__3___redArg___closed__1; if (x_90 == 0) { -x_8 = x_83; -x_9 = x_85; -x_10 = x_88; +x_8 = x_104; +x_9 = x_83; +x_10 = x_85; x_11 = x_108; -x_12 = x_107; -x_13 = x_104; -x_14 = x_105; +x_12 = x_88; +x_13 = x_105; +x_14 = x_107; x_15 = x_6; x_16 = lean_box(0); goto block_81; @@ -45100,13 +45100,13 @@ return x_114; } else { -x_8 = x_83; -x_9 = x_85; -x_10 = x_88; +x_8 = x_104; +x_9 = x_83; +x_10 = x_85; x_11 = x_108; -x_12 = x_107; -x_13 = x_104; -x_14 = x_105; +x_12 = x_88; +x_13 = x_105; +x_14 = x_107; x_15 = x_6; x_16 = lean_box(0); goto block_81; @@ -45117,8 +45117,8 @@ goto block_81; block_124: { lean_object* x_122; -x_122 = l_Lean_Syntax_getTailPos_x3f(x_117, x_120); -lean_dec(x_117); +x_122 = l_Lean_Syntax_getTailPos_x3f(x_119, x_118); +lean_dec(x_119); if (lean_obj_tag(x_122) == 0) { lean_inc(x_121); @@ -45157,16 +45157,16 @@ lean_inc(x_130); lean_dec_ref(x_129); x_131 = l_Lean_replaceRef(x_1, x_130); lean_dec(x_130); -x_132 = l_Lean_Syntax_getPos_x3f(x_131, x_126); +x_132 = l_Lean_Syntax_getPos_x3f(x_131, x_127); if (lean_obj_tag(x_132) == 0) { lean_object* x_133; x_133 = lean_unsigned_to_nat(0u); x_116 = x_125; -x_117 = x_131; -x_118 = x_128; -x_119 = lean_box(0); -x_120 = x_126; +x_117 = lean_box(0); +x_118 = x_127; +x_119 = x_131; +x_120 = x_128; x_121 = x_133; goto block_124; } @@ -45177,10 +45177,10 @@ x_134 = lean_ctor_get(x_132, 0); lean_inc(x_134); lean_dec_ref(x_132); x_116 = x_125; -x_117 = x_131; -x_118 = x_128; -x_119 = lean_box(0); -x_120 = x_126; +x_117 = lean_box(0); +x_118 = x_127; +x_119 = x_131; +x_120 = x_128; x_121 = x_134; goto block_124; } @@ -45212,16 +45212,16 @@ return x_137; if (x_143 == 0) { x_125 = x_140; -x_126 = x_141; -x_127 = lean_box(0); +x_126 = lean_box(0); +x_127 = x_142; x_128 = x_3; goto block_138; } else { x_125 = x_140; -x_126 = x_141; -x_127 = lean_box(0); +x_126 = lean_box(0); +x_127 = x_142; x_128 = x_139; goto block_138; } @@ -45247,8 +45247,8 @@ if (x_152 == 0) { lean_dec(x_150); x_140 = x_145; -x_141 = x_145; -x_142 = lean_box(0); +x_141 = lean_box(0); +x_142 = x_145; x_143 = x_152; goto block_144; } @@ -45259,8 +45259,8 @@ x_153 = l_Lean_logAt___at___00Lean_log___at___00Lean_logWarning___at___00Lean_ch x_154 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Doc_checkNameExists_spec__0_spec__0_spec__1(x_150, x_153); lean_dec(x_150); x_140 = x_145; -x_141 = x_145; -x_142 = lean_box(0); +x_141 = lean_box(0); +x_142 = x_145; x_143 = x_154; goto block_144; } @@ -46273,8 +46273,8 @@ return x_12; { lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; x_23 = lean_alloc_ctor(1, 2, 1); -lean_ctor_set(x_23, 0, x_19); -lean_ctor_set(x_23, 1, x_20); +lean_ctor_set(x_23, 0, x_20); +lean_ctor_set(x_23, 1, x_19); lean_ctor_set_uint8(x_23, sizeof(void*)*2, x_18); lean_inc_ref(x_22); x_24 = l_Lean_Syntax_mkStrLit(x_22, x_23); @@ -46376,8 +46376,8 @@ x_54 = l___private_Lean_Elab_DocString_Builtin_0__Lean_Doc_lean_flagHint___redAr x_55 = lean_nat_dec_le(x_54, x_53); if (x_55 == 0) { -x_19 = x_46; -x_20 = x_47; +x_19 = x_47; +x_20 = x_46; x_21 = lean_box(0); x_22 = x_51; goto block_43; @@ -46389,8 +46389,8 @@ x_56 = lean_unsigned_to_nat(0u); x_57 = lean_string_memcmp(x_51, x_52, x_56, x_56, x_54); if (x_57 == 0) { -x_19 = x_46; -x_20 = x_47; +x_19 = x_47; +x_20 = x_46; x_21 = lean_box(0); x_22 = x_51; goto block_43; @@ -46412,8 +46412,8 @@ lean_dec(x_61); lean_dec_ref(x_51); x_63 = lean_string_append(x_58, x_62); lean_dec_ref(x_62); -x_19 = x_46; -x_20 = x_47; +x_19 = x_47; +x_20 = x_46; x_21 = lean_box(0); x_22 = x_63; goto block_43; @@ -48559,7 +48559,7 @@ return x_43; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; 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; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_110; lean_object* x_111; uint8_t 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_137; lean_object* x_138; lean_object* x_139; uint8_t 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_157; lean_object* x_158; uint8_t 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_184; lean_object* x_185; lean_object* x_186; +lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_110; lean_object* x_111; uint8_t 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_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; uint8_t 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_157; lean_object* x_158; uint8_t 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_184; lean_object* x_185; lean_object* x_186; x_44 = lean_array_uget(x_9, x_11); x_45 = lean_ctor_get(x_44, 1); lean_inc_ref(x_45); @@ -48595,16 +48595,16 @@ goto block_199; { lean_object* x_64; lean_object* x_65; x_64 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_64, 0, x_52); +lean_ctor_set(x_64, 0, x_50); lean_ctor_set(x_64, 1, x_63); -lean_inc(x_57); -lean_inc_ref(x_50); lean_inc(x_62); -lean_inc_ref(x_53); -lean_inc(x_60); -lean_inc_ref(x_58); -x_65 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_55, x_64, x_54, x_58, x_60, x_53, x_62, x_50, x_57); -lean_dec(x_55); +lean_inc_ref(x_54); +lean_inc(x_61); +lean_inc_ref(x_59); +lean_inc(x_55); +lean_inc_ref(x_57); +x_65 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_58, x_64, x_60, x_57, x_55, x_59, x_61, x_54, x_62); +lean_dec(x_58); if (lean_obj_tag(x_65) == 0) { lean_object* x_66; lean_object* x_67; @@ -48613,7 +48613,7 @@ lean_inc(x_66); lean_dec_ref(x_65); lean_inc(x_5); lean_inc(x_4); -x_67 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_51, x_66, x_61, x_56, x_54, x_58, x_60, x_53, x_62, x_50, x_57); +x_67 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_53, x_66, x_51, x_56, x_60, x_57, x_55, x_59, x_61, x_54, x_62); x_23 = x_67; goto block_41; } @@ -48621,12 +48621,12 @@ else { uint8_t x_68; lean_dec(x_62); -lean_dec(x_60); -lean_dec_ref(x_58); -lean_dec(x_57); +lean_dec(x_61); +lean_dec_ref(x_59); +lean_dec_ref(x_57); +lean_dec(x_55); +lean_dec_ref(x_54); lean_dec_ref(x_53); -lean_dec_ref(x_51); -lean_dec_ref(x_50); lean_dec(x_21); lean_dec_ref(x_20); lean_dec(x_19); @@ -48655,25 +48655,25 @@ return x_70; block_109: { 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; uint8_t x_96; lean_object* x_97; uint8_t x_98; lean_object* x_99; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_84 = lean_ctor_get(x_73, 0); -x_85 = lean_ctor_get(x_73, 1); -x_86 = lean_ctor_get(x_73, 2); -x_87 = lean_ctor_get(x_73, 3); -x_88 = lean_ctor_get(x_73, 4); -x_89 = lean_ctor_get(x_73, 5); -x_90 = lean_ctor_get(x_73, 6); -x_91 = lean_ctor_get(x_73, 7); -x_92 = lean_ctor_get(x_73, 8); -x_93 = lean_ctor_get(x_73, 9); -x_94 = lean_ctor_get(x_73, 10); -x_95 = lean_ctor_get(x_73, 11); -x_96 = lean_ctor_get_uint8(x_73, sizeof(void*)*14); -x_97 = lean_ctor_get(x_73, 12); -x_98 = lean_ctor_get_uint8(x_73, sizeof(void*)*14 + 1); -x_99 = lean_ctor_get(x_73, 13); +x_84 = lean_ctor_get(x_76, 0); +x_85 = lean_ctor_get(x_76, 1); +x_86 = lean_ctor_get(x_76, 2); +x_87 = lean_ctor_get(x_76, 3); +x_88 = lean_ctor_get(x_76, 4); +x_89 = lean_ctor_get(x_76, 5); +x_90 = lean_ctor_get(x_76, 6); +x_91 = lean_ctor_get(x_76, 7); +x_92 = lean_ctor_get(x_76, 8); +x_93 = lean_ctor_get(x_76, 9); +x_94 = lean_ctor_get(x_76, 10); +x_95 = lean_ctor_get(x_76, 11); +x_96 = lean_ctor_get_uint8(x_76, sizeof(void*)*14); +x_97 = lean_ctor_get(x_76, 12); +x_98 = lean_ctor_get_uint8(x_76, sizeof(void*)*14 + 1); +x_99 = lean_ctor_get(x_76, 13); x_100 = 0; -x_101 = l_Lean_replaceRef(x_82, x_89); -lean_dec(x_82); +x_101 = l_Lean_replaceRef(x_74, x_89); +lean_dec(x_74); lean_inc_ref(x_99); lean_inc(x_97); lean_inc(x_95); @@ -48704,12 +48704,12 @@ lean_ctor_set(x_102, 12, x_97); lean_ctor_set(x_102, 13, x_99); lean_ctor_set_uint8(x_102, sizeof(void*)*14, x_96); lean_ctor_set_uint8(x_102, sizeof(void*)*14 + 1, x_98); -lean_inc(x_74); lean_inc(x_83); -lean_inc_ref(x_75); -lean_inc(x_79); -lean_inc_ref(x_76); -x_103 = l_Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00Lean_unresolveNameGlobal___at___00Lean_unresolveNameGlobalAvoidingLocals___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_getQualified_spec__0_spec__1_spec__9_spec__19_spec__24_spec__28(x_49, x_100, x_3, x_80, x_81, x_77, x_76, x_79, x_75, x_83, x_102, x_74); +lean_inc(x_80); +lean_inc_ref(x_77); +lean_inc(x_78); +lean_inc_ref(x_82); +x_103 = l_Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00Lean_unresolveNameGlobal___at___00Lean_unresolveNameGlobalAvoidingLocals___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_getQualified_spec__0_spec__1_spec__9_spec__19_spec__24_spec__28(x_49, x_100, x_3, x_73, x_79, x_81, x_82, x_78, x_77, x_80, x_102, x_83); if (lean_obj_tag(x_103) == 0) { lean_object* x_104; lean_object* x_105; @@ -48718,7 +48718,7 @@ lean_inc(x_104); lean_dec_ref(x_103); lean_inc(x_5); lean_inc(x_4); -x_105 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_72, x_104, x_80, x_81, x_77, x_76, x_79, x_75, x_83, x_73, x_74); +x_105 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_75, x_104, x_73, x_79, x_81, x_82, x_78, x_77, x_80, x_76, x_83); x_23 = x_105; goto block_41; } @@ -48726,12 +48726,12 @@ else { uint8_t x_106; lean_dec(x_83); -lean_dec(x_79); +lean_dec_ref(x_82); +lean_dec(x_80); +lean_dec(x_78); +lean_dec_ref(x_77); lean_dec_ref(x_76); lean_dec_ref(x_75); -lean_dec(x_74); -lean_dec_ref(x_73); -lean_dec_ref(x_72); lean_dec(x_21); lean_dec_ref(x_20); lean_dec(x_19); @@ -48764,18 +48764,18 @@ x_122 = 1; x_123 = l_Lean_instBEqMessageSeverity_beq(x_47, x_122); if (x_123 == 0) { -x_72 = x_110; -x_73 = x_119; -x_74 = x_120; -x_75 = x_117; -x_76 = x_115; -x_77 = x_114; -x_78 = lean_box(0); -x_79 = x_116; -x_80 = x_112; -x_81 = x_113; -x_82 = x_111; -x_83 = x_118; +x_72 = lean_box(0); +x_73 = x_112; +x_74 = x_110; +x_75 = x_111; +x_76 = x_119; +x_77 = x_117; +x_78 = x_116; +x_79 = x_113; +x_80 = x_118; +x_81 = x_114; +x_82 = x_115; +x_83 = x_120; goto block_109; } else @@ -48784,18 +48784,18 @@ if (x_6 == 0) { if (x_123 == 0) { -x_72 = x_110; -x_73 = x_119; -x_74 = x_120; -x_75 = x_117; -x_76 = x_115; -x_77 = x_114; -x_78 = lean_box(0); -x_79 = x_116; -x_80 = x_112; -x_81 = x_113; -x_82 = x_111; -x_83 = x_118; +x_72 = lean_box(0); +x_73 = x_112; +x_74 = x_110; +x_75 = x_111; +x_76 = x_119; +x_77 = x_117; +x_78 = x_116; +x_79 = x_113; +x_80 = x_118; +x_81 = x_114; +x_82 = x_115; +x_83 = x_120; goto block_109; } else @@ -48825,19 +48825,19 @@ if (lean_obj_tag(x_127) == 0) { lean_object* x_131; x_131 = l___private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_elabExtraTerm_spec__0_spec__0___closed__14; -x_50 = x_119; -x_51 = x_110; -x_52 = x_130; -x_53 = x_117; -x_54 = x_114; -x_55 = x_111; +x_50 = x_130; +x_51 = x_112; +x_52 = lean_box(0); +x_53 = x_111; +x_54 = x_119; +x_55 = x_116; x_56 = x_113; -x_57 = x_120; -x_58 = x_115; -x_59 = lean_box(0); -x_60 = x_116; -x_61 = x_112; -x_62 = x_118; +x_57 = x_115; +x_58 = x_110; +x_59 = x_117; +x_60 = x_114; +x_61 = x_118; +x_62 = x_120; x_63 = x_131; goto block_71; } @@ -48847,19 +48847,19 @@ lean_object* x_132; x_132 = lean_ctor_get(x_127, 0); lean_inc(x_132); lean_dec_ref(x_127); -x_50 = x_119; -x_51 = x_110; -x_52 = x_130; -x_53 = x_117; -x_54 = x_114; -x_55 = x_111; +x_50 = x_130; +x_51 = x_112; +x_52 = lean_box(0); +x_53 = x_111; +x_54 = x_119; +x_55 = x_116; x_56 = x_113; -x_57 = x_120; -x_58 = x_115; -x_59 = lean_box(0); -x_60 = x_116; -x_61 = x_112; -x_62 = x_118; +x_57 = x_115; +x_58 = x_110; +x_59 = x_117; +x_60 = x_114; +x_61 = x_118; +x_62 = x_120; x_63 = x_132; goto block_71; } @@ -48873,8 +48873,8 @@ lean_dec(x_118); lean_dec_ref(x_117); lean_dec(x_116); lean_dec_ref(x_115); -lean_dec(x_111); -lean_dec_ref(x_110); +lean_dec_ref(x_111); +lean_dec(x_110); lean_dec(x_49); lean_dec(x_21); lean_dec_ref(x_20); @@ -48904,18 +48904,18 @@ return x_135; } else { -x_72 = x_110; -x_73 = x_119; -x_74 = x_120; -x_75 = x_117; -x_76 = x_115; -x_77 = x_114; -x_78 = lean_box(0); -x_79 = x_116; -x_80 = x_112; -x_81 = x_113; -x_82 = x_111; -x_83 = x_118; +x_72 = lean_box(0); +x_73 = x_112; +x_74 = x_110; +x_75 = x_111; +x_76 = x_119; +x_77 = x_117; +x_78 = x_116; +x_79 = x_113; +x_80 = x_118; +x_81 = x_114; +x_82 = x_115; +x_83 = x_120; goto block_109; } } @@ -48924,43 +48924,43 @@ goto block_109; { lean_object* x_151; lean_object* x_152; x_151 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_151, 0, x_145); +lean_ctor_set(x_151, 0, x_149); lean_ctor_set(x_151, 1, x_150); -lean_inc(x_138); -lean_inc_ref(x_148); -lean_inc(x_149); -lean_inc_ref(x_147); -lean_inc(x_143); +lean_inc(x_147); lean_inc_ref(x_144); -x_152 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_146, x_151, x_141, x_144, x_143, x_147, x_149, x_148, x_138); +lean_inc(x_142); +lean_inc_ref(x_143); +lean_inc(x_141); +lean_inc_ref(x_140); +x_152 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_146, x_151, x_138, x_140, x_141, x_143, x_142, x_144, x_147); if (lean_obj_tag(x_152) == 0) { lean_dec_ref(x_152); -x_110 = x_137; -x_111 = x_146; -x_112 = x_140; -x_113 = x_142; -x_114 = x_141; -x_115 = x_144; -x_116 = x_143; -x_117 = x_147; -x_118 = x_149; -x_119 = x_148; -x_120 = x_138; +x_110 = x_146; +x_111 = x_139; +x_112 = x_145; +x_113 = x_137; +x_114 = x_138; +x_115 = x_140; +x_116 = x_141; +x_117 = x_143; +x_118 = x_142; +x_119 = x_144; +x_120 = x_147; x_121 = lean_box(0); goto block_136; } else { uint8_t x_153; -lean_dec(x_149); -lean_dec_ref(x_148); -lean_dec_ref(x_147); +lean_dec(x_147); lean_dec(x_146); lean_dec_ref(x_144); -lean_dec(x_143); -lean_dec(x_138); -lean_dec_ref(x_137); +lean_dec_ref(x_143); +lean_dec(x_142); +lean_dec(x_141); +lean_dec_ref(x_140); +lean_dec_ref(x_139); lean_dec(x_49); lean_dec(x_21); lean_dec_ref(x_20); @@ -48994,8 +48994,8 @@ x_169 = 2; x_170 = l_Lean_instBEqMessageSeverity_beq(x_47, x_169); if (x_170 == 0) { -x_110 = x_158; -x_111 = x_157; +x_110 = x_157; +x_111 = x_158; x_112 = x_159; x_113 = x_160; x_114 = x_161; @@ -49014,8 +49014,8 @@ if (x_7 == 0) { if (x_170 == 0) { -x_110 = x_158; -x_111 = x_157; +x_110 = x_157; +x_111 = x_158; x_112 = x_159; x_113 = x_160; x_114 = x_161; @@ -49056,19 +49056,19 @@ if (lean_obj_tag(x_174) == 0) { lean_object* x_178; x_178 = l___private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_elabExtraTerm_spec__0_spec__0___closed__14; -x_137 = x_158; -x_138 = x_167; -x_139 = lean_box(0); -x_140 = x_159; -x_141 = x_161; -x_142 = x_160; -x_143 = x_163; -x_144 = x_162; -x_145 = x_177; +x_137 = x_160; +x_138 = x_161; +x_139 = x_158; +x_140 = x_162; +x_141 = x_163; +x_142 = x_165; +x_143 = x_164; +x_144 = x_166; +x_145 = x_159; x_146 = x_157; -x_147 = x_164; -x_148 = x_166; -x_149 = x_165; +x_147 = x_167; +x_148 = lean_box(0); +x_149 = x_177; x_150 = x_178; goto block_156; } @@ -49078,19 +49078,19 @@ lean_object* x_179; x_179 = lean_ctor_get(x_174, 0); lean_inc(x_179); lean_dec_ref(x_174); -x_137 = x_158; -x_138 = x_167; -x_139 = lean_box(0); -x_140 = x_159; -x_141 = x_161; -x_142 = x_160; -x_143 = x_163; -x_144 = x_162; -x_145 = x_177; +x_137 = x_160; +x_138 = x_161; +x_139 = x_158; +x_140 = x_162; +x_141 = x_163; +x_142 = x_165; +x_143 = x_164; +x_144 = x_166; +x_145 = x_159; x_146 = x_157; -x_147 = x_164; -x_148 = x_166; -x_149 = x_165; +x_147 = x_167; +x_148 = lean_box(0); +x_149 = x_177; x_150 = x_179; goto block_156; } @@ -49135,8 +49135,8 @@ return x_182; } else { -x_110 = x_158; -x_111 = x_157; +x_110 = x_157; +x_111 = x_158; x_112 = x_159; x_113 = x_160; x_114 = x_161; @@ -49410,7 +49410,7 @@ return x_43; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_110; lean_object* x_111; uint8_t 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_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_157; lean_object* x_158; uint8_t 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_184; lean_object* x_185; lean_object* x_186; +lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; 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; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_110; lean_object* x_111; uint8_t 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_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; uint8_t x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_157; lean_object* x_158; uint8_t 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_184; lean_object* x_185; lean_object* x_186; x_44 = lean_array_uget(x_9, x_11); x_45 = lean_ctor_get(x_44, 1); lean_inc_ref(x_45); @@ -49446,16 +49446,16 @@ goto block_199; { lean_object* x_64; lean_object* x_65; x_64 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 0, x_50); lean_ctor_set(x_64, 1, x_63); -lean_inc(x_57); -lean_inc_ref(x_60); -lean_inc(x_58); -lean_inc_ref(x_53); -lean_inc(x_51); -lean_inc_ref(x_50); -x_65 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_59, x_64, x_54, x_50, x_51, x_53, x_58, x_60, x_57); -lean_dec(x_59); +lean_inc(x_60); +lean_inc_ref(x_55); +lean_inc(x_52); +lean_inc_ref(x_51); +lean_inc(x_56); +lean_inc_ref(x_59); +x_65 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_61, x_64, x_53, x_59, x_56, x_51, x_52, x_55, x_60); +lean_dec(x_61); if (lean_obj_tag(x_65) == 0) { lean_object* x_66; lean_object* x_67; @@ -49464,20 +49464,20 @@ lean_inc(x_66); lean_dec_ref(x_65); lean_inc(x_5); lean_inc(x_4); -x_67 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_55, x_66, x_52, x_56, x_54, x_50, x_51, x_53, x_58, x_60, x_57); +x_67 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_58, x_66, x_62, x_54, x_53, x_59, x_56, x_51, x_52, x_55, x_60); x_23 = x_67; goto block_41; } else { uint8_t x_68; -lean_dec_ref(x_60); -lean_dec(x_58); -lean_dec(x_57); +lean_dec(x_60); +lean_dec_ref(x_59); +lean_dec_ref(x_58); +lean_dec(x_56); lean_dec_ref(x_55); -lean_dec_ref(x_53); -lean_dec(x_51); -lean_dec_ref(x_50); +lean_dec(x_52); +lean_dec_ref(x_51); lean_dec(x_21); lean_dec_ref(x_20); lean_dec(x_19); @@ -49506,25 +49506,25 @@ return x_70; block_109: { 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; uint8_t x_96; lean_object* x_97; uint8_t x_98; lean_object* x_99; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_84 = lean_ctor_get(x_79, 0); -x_85 = lean_ctor_get(x_79, 1); -x_86 = lean_ctor_get(x_79, 2); -x_87 = lean_ctor_get(x_79, 3); -x_88 = lean_ctor_get(x_79, 4); -x_89 = lean_ctor_get(x_79, 5); -x_90 = lean_ctor_get(x_79, 6); -x_91 = lean_ctor_get(x_79, 7); -x_92 = lean_ctor_get(x_79, 8); -x_93 = lean_ctor_get(x_79, 9); -x_94 = lean_ctor_get(x_79, 10); -x_95 = lean_ctor_get(x_79, 11); -x_96 = lean_ctor_get_uint8(x_79, sizeof(void*)*14); -x_97 = lean_ctor_get(x_79, 12); -x_98 = lean_ctor_get_uint8(x_79, sizeof(void*)*14 + 1); -x_99 = lean_ctor_get(x_79, 13); +x_84 = lean_ctor_get(x_78, 0); +x_85 = lean_ctor_get(x_78, 1); +x_86 = lean_ctor_get(x_78, 2); +x_87 = lean_ctor_get(x_78, 3); +x_88 = lean_ctor_get(x_78, 4); +x_89 = lean_ctor_get(x_78, 5); +x_90 = lean_ctor_get(x_78, 6); +x_91 = lean_ctor_get(x_78, 7); +x_92 = lean_ctor_get(x_78, 8); +x_93 = lean_ctor_get(x_78, 9); +x_94 = lean_ctor_get(x_78, 10); +x_95 = lean_ctor_get(x_78, 11); +x_96 = lean_ctor_get_uint8(x_78, sizeof(void*)*14); +x_97 = lean_ctor_get(x_78, 12); +x_98 = lean_ctor_get_uint8(x_78, sizeof(void*)*14 + 1); +x_99 = lean_ctor_get(x_78, 13); x_100 = 0; -x_101 = l_Lean_replaceRef(x_78, x_89); -lean_dec(x_78); +x_101 = l_Lean_replaceRef(x_77, x_89); +lean_dec(x_77); lean_inc_ref(x_99); lean_inc(x_97); lean_inc(x_95); @@ -49555,12 +49555,12 @@ lean_ctor_set(x_102, 12, x_97); lean_ctor_set(x_102, 13, x_99); lean_ctor_set_uint8(x_102, sizeof(void*)*14, x_96); lean_ctor_set_uint8(x_102, sizeof(void*)*14 + 1, x_98); -lean_inc(x_72); -lean_inc(x_76); -lean_inc_ref(x_77); -lean_inc(x_74); -lean_inc_ref(x_73); -x_103 = l_Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00Lean_unresolveNameGlobal___at___00Lean_unresolveNameGlobalAvoidingLocals___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_getQualified_spec__0_spec__1_spec__9_spec__19_spec__24_spec__28(x_49, x_100, x_3, x_75, x_83, x_81, x_73, x_74, x_77, x_76, x_102, x_72); +lean_inc(x_75); +lean_inc(x_73); +lean_inc_ref(x_72); +lean_inc(x_81); +lean_inc_ref(x_83); +x_103 = l_Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00Lean_unresolveNameGlobal___at___00Lean_unresolveNameGlobalAvoidingLocals___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_getQualified_spec__0_spec__1_spec__9_spec__19_spec__24_spec__28(x_49, x_100, x_3, x_80, x_76, x_74, x_83, x_81, x_72, x_73, x_102, x_75); if (lean_obj_tag(x_103) == 0) { lean_object* x_104; lean_object* x_105; @@ -49569,20 +49569,20 @@ lean_inc(x_104); lean_dec_ref(x_103); lean_inc(x_5); lean_inc(x_4); -x_105 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_80, x_104, x_75, x_83, x_81, x_73, x_74, x_77, x_76, x_79, x_72); +x_105 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Doc_lean_spec__3___redArg___lam__2(x_4, x_5, x_82, x_104, x_80, x_76, x_74, x_83, x_81, x_72, x_73, x_78, x_75); x_23 = x_105; goto block_41; } else { uint8_t x_106; -lean_dec_ref(x_80); -lean_dec_ref(x_79); -lean_dec_ref(x_77); -lean_dec(x_76); -lean_dec(x_74); -lean_dec_ref(x_73); -lean_dec(x_72); +lean_dec_ref(x_83); +lean_dec_ref(x_82); +lean_dec(x_81); +lean_dec_ref(x_78); +lean_dec(x_75); +lean_dec(x_73); +lean_dec_ref(x_72); lean_dec(x_21); lean_dec_ref(x_20); lean_dec(x_19); @@ -49615,18 +49615,18 @@ x_122 = 1; x_123 = l_Lean_instBEqMessageSeverity_beq(x_47, x_122); if (x_123 == 0) { -x_72 = x_120; -x_73 = x_115; -x_74 = x_116; -x_75 = x_112; -x_76 = x_118; -x_77 = x_117; -x_78 = x_110; -x_79 = x_119; -x_80 = x_111; -x_81 = x_114; -x_82 = lean_box(0); -x_83 = x_113; +x_72 = x_117; +x_73 = x_118; +x_74 = x_114; +x_75 = x_120; +x_76 = x_113; +x_77 = x_110; +x_78 = x_119; +x_79 = lean_box(0); +x_80 = x_112; +x_81 = x_116; +x_82 = x_111; +x_83 = x_115; goto block_109; } else @@ -49635,18 +49635,18 @@ if (x_6 == 0) { if (x_123 == 0) { -x_72 = x_120; -x_73 = x_115; -x_74 = x_116; -x_75 = x_112; -x_76 = x_118; -x_77 = x_117; -x_78 = x_110; -x_79 = x_119; -x_80 = x_111; -x_81 = x_114; -x_82 = lean_box(0); -x_83 = x_113; +x_72 = x_117; +x_73 = x_118; +x_74 = x_114; +x_75 = x_120; +x_76 = x_113; +x_77 = x_110; +x_78 = x_119; +x_79 = lean_box(0); +x_80 = x_112; +x_81 = x_116; +x_82 = x_111; +x_83 = x_115; goto block_109; } else @@ -49676,19 +49676,19 @@ if (lean_obj_tag(x_127) == 0) { lean_object* x_131; x_131 = l___private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_elabExtraTerm_spec__0_spec__0___closed__14; -x_50 = x_115; -x_51 = x_116; -x_52 = x_112; -x_53 = x_117; -x_54 = x_114; -x_55 = x_111; -x_56 = x_113; -x_57 = x_120; -x_58 = x_118; -x_59 = x_110; -x_60 = x_119; -x_61 = x_130; -x_62 = lean_box(0); +x_50 = x_130; +x_51 = x_117; +x_52 = x_118; +x_53 = x_114; +x_54 = x_113; +x_55 = x_119; +x_56 = x_116; +x_57 = lean_box(0); +x_58 = x_111; +x_59 = x_115; +x_60 = x_120; +x_61 = x_110; +x_62 = x_112; x_63 = x_131; goto block_71; } @@ -49698,19 +49698,19 @@ lean_object* x_132; x_132 = lean_ctor_get(x_127, 0); lean_inc(x_132); lean_dec_ref(x_127); -x_50 = x_115; -x_51 = x_116; -x_52 = x_112; -x_53 = x_117; -x_54 = x_114; -x_55 = x_111; -x_56 = x_113; -x_57 = x_120; -x_58 = x_118; -x_59 = x_110; -x_60 = x_119; -x_61 = x_130; -x_62 = lean_box(0); +x_50 = x_130; +x_51 = x_117; +x_52 = x_118; +x_53 = x_114; +x_54 = x_113; +x_55 = x_119; +x_56 = x_116; +x_57 = lean_box(0); +x_58 = x_111; +x_59 = x_115; +x_60 = x_120; +x_61 = x_110; +x_62 = x_112; x_63 = x_132; goto block_71; } @@ -49755,18 +49755,18 @@ return x_135; } else { -x_72 = x_120; -x_73 = x_115; -x_74 = x_116; -x_75 = x_112; -x_76 = x_118; -x_77 = x_117; -x_78 = x_110; -x_79 = x_119; -x_80 = x_111; -x_81 = x_114; -x_82 = lean_box(0); -x_83 = x_113; +x_72 = x_117; +x_73 = x_118; +x_74 = x_114; +x_75 = x_120; +x_76 = x_113; +x_77 = x_110; +x_78 = x_119; +x_79 = lean_box(0); +x_80 = x_112; +x_81 = x_116; +x_82 = x_111; +x_83 = x_115; goto block_109; } } @@ -49775,29 +49775,29 @@ goto block_109; { lean_object* x_151; lean_object* x_152; x_151 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_151, 0, x_146); +lean_ctor_set(x_151, 0, x_142); lean_ctor_set(x_151, 1, x_150); -lean_inc(x_145); -lean_inc_ref(x_140); -lean_inc(x_139); -lean_inc_ref(x_142); +lean_inc(x_140); +lean_inc_ref(x_145); lean_inc(x_149); -lean_inc_ref(x_137); -x_152 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_144, x_151, x_147, x_137, x_149, x_142, x_139, x_140, x_145); +lean_inc_ref(x_138); +lean_inc(x_148); +lean_inc_ref(x_146); +x_152 = l_Lean_logErrorAt___at___00Lean_Doc_name_spec__2___redArg(x_144, x_151, x_143, x_146, x_148, x_138, x_149, x_145, x_140); if (lean_obj_tag(x_152) == 0) { lean_dec_ref(x_152); x_110 = x_144; -x_111 = x_138; -x_112 = x_141; -x_113 = x_143; -x_114 = x_147; -x_115 = x_137; -x_116 = x_149; -x_117 = x_142; -x_118 = x_139; -x_119 = x_140; -x_120 = x_145; +x_111 = x_141; +x_112 = x_147; +x_113 = x_139; +x_114 = x_143; +x_115 = x_146; +x_116 = x_148; +x_117 = x_138; +x_118 = x_149; +x_119 = x_145; +x_120 = x_140; x_121 = lean_box(0); goto block_136; } @@ -49805,13 +49805,13 @@ else { uint8_t x_153; lean_dec(x_149); -lean_dec(x_145); +lean_dec(x_148); +lean_dec_ref(x_146); +lean_dec_ref(x_145); lean_dec(x_144); -lean_dec_ref(x_142); -lean_dec_ref(x_140); -lean_dec(x_139); +lean_dec_ref(x_141); +lean_dec(x_140); lean_dec_ref(x_138); -lean_dec_ref(x_137); lean_dec(x_49); lean_dec(x_21); lean_dec_ref(x_20); @@ -49907,19 +49907,19 @@ if (lean_obj_tag(x_174) == 0) { lean_object* x_178; x_178 = l___private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00__private_Lean_Elab_DocString_Builtin_0__Lean_Doc_elabExtraTerm_spec__0_spec__0___closed__14; -x_137 = x_162; -x_138 = x_158; -x_139 = x_165; -x_140 = x_166; -x_141 = x_159; -x_142 = x_164; -x_143 = x_160; +x_137 = lean_box(0); +x_138 = x_164; +x_139 = x_160; +x_140 = x_167; +x_141 = x_158; +x_142 = x_177; +x_143 = x_161; x_144 = x_157; -x_145 = x_167; -x_146 = x_177; -x_147 = x_161; -x_148 = lean_box(0); -x_149 = x_163; +x_145 = x_166; +x_146 = x_162; +x_147 = x_159; +x_148 = x_163; +x_149 = x_165; x_150 = x_178; goto block_156; } @@ -49929,19 +49929,19 @@ lean_object* x_179; x_179 = lean_ctor_get(x_174, 0); lean_inc(x_179); lean_dec_ref(x_174); -x_137 = x_162; -x_138 = x_158; -x_139 = x_165; -x_140 = x_166; -x_141 = x_159; -x_142 = x_164; -x_143 = x_160; +x_137 = lean_box(0); +x_138 = x_164; +x_139 = x_160; +x_140 = x_167; +x_141 = x_158; +x_142 = x_177; +x_143 = x_161; x_144 = x_157; -x_145 = x_167; -x_146 = x_177; -x_147 = x_161; -x_148 = lean_box(0); -x_149 = x_163; +x_145 = x_166; +x_146 = x_162; +x_147 = x_159; +x_148 = x_163; +x_149 = x_165; x_150 = x_179; goto block_156; } @@ -66624,7 +66624,7 @@ lean_dec(x_266); x_312 = l_Lean_Doc_option___closed__8; x_313 = l_Lean_Doc_option___closed__9; x_314 = lean_array_push(x_313, x_265); -x_315 = lean_array_push(x_314, x_310); +x_315 = lean_array_push(x_314, x_309); x_316 = l___private_Lean_Elab_DocString_Builtin_0__Lean_Doc_throwOrNest___redArg(x_312, x_315, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_317 = !lean_is_exclusive(x_316); if (x_317 == 0) @@ -66657,7 +66657,7 @@ if (lean_is_scalar(x_266)) { } else { x_320 = x_266; } -lean_ctor_set(x_320, 0, x_310); +lean_ctor_set(x_320, 0, x_309); return x_320; } } @@ -66670,15 +66670,15 @@ if (x_324 == 0) uint8_t x_325; lean_inc_ref(x_322); x_325 = l_Lean_Exception_isRuntime(x_322); -x_309 = lean_box(0); -x_310 = x_322; +x_309 = x_322; +x_310 = lean_box(0); x_311 = x_325; goto block_321; } else { -x_309 = lean_box(0); -x_310 = x_322; +x_309 = x_322; +x_310 = lean_box(0); x_311 = x_324; goto block_321; } @@ -66875,7 +66875,7 @@ return x_352; if (x_71 == 0) { lean_object* x_72; uint8_t x_73; -lean_dec_ref(x_68); +lean_dec_ref(x_70); x_72 = l_Lean_Exception_getRef(x_69); x_73 = l_Lean_Syntax_isMissing(x_72); if (x_73 == 0) @@ -66920,7 +66920,7 @@ lean_dec(x_8); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_5); -return x_68; +return x_70; } } block_80: @@ -66932,17 +66932,17 @@ if (x_78 == 0) uint8_t x_79; lean_inc_ref(x_76); x_79 = l_Lean_Exception_isRuntime(x_76); -x_68 = x_75; +x_68 = lean_box(0); x_69 = x_76; -x_70 = lean_box(0); +x_70 = x_75; x_71 = x_79; goto block_74; } else { -x_68 = x_75; +x_68 = lean_box(0); x_69 = x_76; -x_70 = lean_box(0); +x_70 = x_75; x_71 = x_78; goto block_74; } @@ -67632,7 +67632,7 @@ return x_248; if (x_253 == 0) { lean_object* x_254; uint8_t x_255; -lean_dec_ref(x_252); +lean_dec_ref(x_251); x_254 = l_Lean_Exception_getRef(x_250); x_255 = l_Lean_Syntax_isMissing(x_254); if (x_255 == 0) @@ -67677,7 +67677,7 @@ lean_dec(x_8); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_5); -return x_252; +return x_251; } } block_262: @@ -67690,16 +67690,16 @@ uint8_t x_261; lean_inc_ref(x_258); x_261 = l_Lean_Exception_isRuntime(x_258); x_250 = x_258; -x_251 = lean_box(0); -x_252 = x_257; +x_251 = x_257; +x_252 = lean_box(0); x_253 = x_261; goto block_256; } else { x_250 = x_258; -x_251 = lean_box(0); -x_252 = x_257; +x_251 = x_257; +x_252 = lean_box(0); x_253 = x_260; goto block_256; } @@ -67952,7 +67952,7 @@ lean_dec(x_477); x_511 = l_Lean_Doc_option___closed__8; x_512 = l_Lean_Doc_option___closed__9; x_513 = lean_array_push(x_512, x_476); -x_514 = lean_array_push(x_513, x_509); +x_514 = lean_array_push(x_513, x_508); x_515 = l___private_Lean_Elab_DocString_Builtin_0__Lean_Doc_throwOrNest___redArg(x_511, x_514, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_374, x_10); x_516 = lean_ctor_get(x_515, 0); lean_inc(x_516); @@ -67986,7 +67986,7 @@ if (lean_is_scalar(x_477)) { } else { x_519 = x_477; } -lean_ctor_set(x_519, 0, x_509); +lean_ctor_set(x_519, 0, x_508); return x_519; } } @@ -67999,15 +67999,15 @@ if (x_523 == 0) uint8_t x_524; lean_inc_ref(x_521); x_524 = l_Lean_Exception_isRuntime(x_521); -x_508 = lean_box(0); -x_509 = x_521; +x_508 = x_521; +x_509 = lean_box(0); x_510 = x_524; goto block_520; } else { -x_508 = lean_box(0); -x_509 = x_521; +x_508 = x_521; +x_509 = lean_box(0); x_510 = x_523; goto block_520; } @@ -68148,7 +68148,7 @@ return x_543; if (x_378 == 0) { lean_object* x_379; uint8_t x_380; -lean_dec_ref(x_375); +lean_dec_ref(x_377); x_379 = l_Lean_Exception_getRef(x_376); x_380 = l_Lean_Syntax_isMissing(x_379); if (x_380 == 0) @@ -68193,7 +68193,7 @@ lean_dec(x_8); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_5); -return x_375; +return x_377; } } block_387: @@ -68205,17 +68205,17 @@ if (x_385 == 0) uint8_t x_386; lean_inc_ref(x_383); x_386 = l_Lean_Exception_isRuntime(x_383); -x_375 = x_382; +x_375 = lean_box(0); x_376 = x_383; -x_377 = lean_box(0); +x_377 = x_382; x_378 = x_386; goto block_381; } else { -x_375 = x_382; +x_375 = lean_box(0); x_376 = x_383; -x_377 = lean_box(0); +x_377 = x_382; x_378 = x_385; goto block_381; } @@ -68564,7 +68564,7 @@ return x_459; if (x_464 == 0) { lean_object* x_465; uint8_t x_466; -lean_dec_ref(x_463); +lean_dec_ref(x_462); x_465 = l_Lean_Exception_getRef(x_461); x_466 = l_Lean_Syntax_isMissing(x_465); if (x_466 == 0) @@ -68609,7 +68609,7 @@ lean_dec(x_8); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_5); -return x_463; +return x_462; } } block_473: @@ -68622,16 +68622,16 @@ uint8_t x_472; lean_inc_ref(x_469); x_472 = l_Lean_Exception_isRuntime(x_469); x_461 = x_469; -x_462 = lean_box(0); -x_463 = x_468; +x_462 = x_468; +x_463 = lean_box(0); x_464 = x_472; goto block_467; } else { x_461 = x_469; -x_462 = lean_box(0); -x_463 = x_468; +x_462 = x_468; +x_463 = lean_box(0); x_464 = x_471; goto block_467; } @@ -81598,7 +81598,7 @@ goto block_23; if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -lean_dec_ref(x_13); +lean_dec_ref(x_12); x_15 = l_Lean_Doc_suggestName___closed__0; x_16 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_16, 0, x_15); @@ -81606,7 +81606,7 @@ return x_16; } else { -return x_13; +return x_12; } } block_23: @@ -81617,16 +81617,16 @@ if (x_21 == 0) { uint8_t x_22; x_22 = l_Lean_Exception_isRuntime(x_19); -x_12 = lean_box(0); -x_13 = x_18; +x_12 = x_18; +x_13 = lean_box(0); x_14 = x_22; goto block_17; } else { lean_dec_ref(x_19); -x_12 = lean_box(0); -x_13 = x_18; +x_12 = x_18; +x_13 = lean_box(0); x_14 = x_21; goto block_17; } @@ -81978,7 +81978,7 @@ goto block_23; if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -lean_dec_ref(x_12); +lean_dec_ref(x_13); x_15 = l_Lean_Doc_suggestLeanTermBlock___closed__0; x_16 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_16, 0, x_15); @@ -81986,7 +81986,7 @@ return x_16; } else { -return x_12; +return x_13; } } block_23: @@ -81997,16 +81997,16 @@ if (x_21 == 0) { uint8_t x_22; x_22 = l_Lean_Exception_isRuntime(x_19); -x_12 = x_18; -x_13 = lean_box(0); +x_12 = lean_box(0); +x_13 = x_18; x_14 = x_22; goto block_17; } else { lean_dec_ref(x_19); -x_12 = x_18; -x_13 = lean_box(0); +x_12 = lean_box(0); +x_13 = x_18; x_14 = x_21; goto block_17; } @@ -83935,7 +83935,7 @@ return x_59; if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -lean_dec_ref(x_13); +lean_dec_ref(x_12); x_15 = l_Lean_Doc_suggestName___closed__0; x_16 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_16, 0, x_15); @@ -83943,7 +83943,7 @@ return x_16; } else { -return x_13; +return x_12; } } block_23: @@ -83954,16 +83954,16 @@ if (x_21 == 0) { uint8_t x_22; x_22 = l_Lean_Exception_isRuntime(x_19); -x_12 = lean_box(0); -x_13 = x_18; +x_12 = x_18; +x_13 = lean_box(0); x_14 = x_22; goto block_17; } else { lean_dec_ref(x_19); -x_12 = lean_box(0); -x_13 = x_18; +x_12 = x_18; +x_13 = lean_box(0); x_14 = x_21; goto block_17; } diff --git a/stage0/stdlib/Lean/Elab/MutualInductive.c b/stage0/stdlib/Lean/Elab/MutualInductive.c index ba0ba2930ff7..a312597d4b79 100644 --- a/stage0/stdlib/Lean/Elab/MutualInductive.c +++ b/stage0/stdlib/Lean/Elab/MutualInductive.c @@ -7080,7 +7080,7 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux___lam__1(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_61; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_61; if (lean_obj_tag(x_5) == 0) { lean_object* x_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; @@ -7146,7 +7146,7 @@ x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); lean_dec_ref(x_26); x_28 = 1; -x_29 = l_Lean_Meta_mkForallFVars(x_27, x_20, x_23, x_1, x_1, x_28, x_8, x_9, x_10, x_11); +x_29 = l_Lean_Meta_mkForallFVars(x_27, x_20, x_21, x_1, x_1, x_28, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_29) == 0) { if (x_2 == 0) @@ -7425,18 +7425,18 @@ if (lean_obj_tag(x_66) == 0) lean_object* x_67; x_67 = l_Lean_Syntax_getTailPos_x3f(x_4, x_1); x_20 = x_63; -x_21 = lean_box(0); +x_21 = x_64; x_22 = x_61; -x_23 = x_64; +x_23 = lean_box(0); x_24 = x_67; goto block_60; } else { x_20 = x_63; -x_21 = lean_box(0); +x_21 = x_64; x_22 = x_61; -x_23 = x_64; +x_23 = lean_box(0); x_24 = x_66; goto block_60; } @@ -11627,29 +11627,29 @@ return x_86; { lean_object* x_19; lean_inc(x_11); -lean_inc_ref(x_13); -lean_inc(x_12); -lean_inc_ref(x_15); +lean_inc_ref(x_12); +lean_inc(x_15); +lean_inc_ref(x_14); lean_inc_ref(x_2); lean_inc_ref(x_1); -x_19 = l___private_Lean_Util_ForEachExprWhere_0__Lean_ForEachExprWhere_visit_go___at___00Lean_ForEachExprWhere_visit___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go_spec__3_spec__3(x_1, x_2, x_3, x_16, x_18, x_15, x_12, x_13, x_11); +x_19 = l___private_Lean_Util_ForEachExprWhere_0__Lean_ForEachExprWhere_visit_go___at___00Lean_ForEachExprWhere_visit___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go_spec__3_spec__3(x_1, x_2, x_3, x_16, x_18, x_14, x_15, x_12, x_11); if (lean_obj_tag(x_19) == 0) { lean_dec_ref(x_19); x_4 = x_17; x_5 = x_18; -x_6 = x_15; -x_7 = x_12; -x_8 = x_13; +x_6 = x_14; +x_7 = x_15; +x_8 = x_12; x_9 = x_11; goto _start; } else { lean_dec_ref(x_17); -lean_dec_ref(x_15); -lean_dec_ref(x_13); -lean_dec(x_12); +lean_dec(x_15); +lean_dec_ref(x_14); +lean_dec_ref(x_12); lean_dec(x_11); lean_dec_ref(x_2); lean_dec_ref(x_1); @@ -11668,10 +11668,10 @@ x_29 = lean_ctor_get(x_4, 2); lean_inc_ref(x_29); lean_dec_ref(x_4); x_11 = x_26; -x_12 = x_24; -x_13 = x_25; -x_14 = lean_box(0); -x_15 = x_23; +x_12 = x_25; +x_13 = lean_box(0); +x_14 = x_23; +x_15 = x_24; x_16 = x_28; x_17 = x_29; x_18 = x_22; @@ -11686,10 +11686,10 @@ x_31 = lean_ctor_get(x_4, 2); lean_inc_ref(x_31); lean_dec_ref(x_4); x_11 = x_26; -x_12 = x_24; -x_13 = x_25; -x_14 = lean_box(0); -x_15 = x_23; +x_12 = x_25; +x_13 = lean_box(0); +x_14 = x_23; +x_15 = x_24; x_16 = x_30; x_17 = x_31; x_18 = x_22; @@ -17270,12 +17270,12 @@ goto _start; if (x_17 == 0) { uint8_t x_18; -x_18 = l_Lean_Level_occurs(x_1, x_14); +x_18 = l_Lean_Level_occurs(x_1, x_16); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_1); -x_19 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_AccLevelState_push(x_16, x_14, x_15); +x_19 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_AccLevelState_push(x_14, x_16, x_15); x_20 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_accLevel_go___closed__0; x_21 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_21, 0, x_20); @@ -17286,7 +17286,7 @@ else { lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; x_22 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_accLevel_go___closed__2; -x_23 = l_Lean_MessageData_ofLevel(x_14); +x_23 = l_Lean_MessageData_ofLevel(x_16); x_24 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_24, 0, x_22); lean_ctor_set(x_24, 1, x_23); @@ -17316,20 +17316,20 @@ x_36 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_36, 0, 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_16); +lean_ctor_set(x_37, 1, x_14); return x_37; } } else { lean_object* x_38; lean_object* x_39; +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_1); x_38 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_accLevel_go___closed__0; x_39 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_16); +lean_ctor_set(x_39, 1, x_14); return x_39; } } @@ -17339,9 +17339,9 @@ uint8_t x_44; x_44 = lean_level_eq(x_41, x_1); if (x_44 == 0) { -x_14 = x_41; +x_14 = x_43; x_15 = x_42; -x_16 = x_43; +x_16 = x_41; x_17 = x_44; goto block_40; } @@ -17350,9 +17350,9 @@ else lean_object* x_45; uint8_t x_46; x_45 = lean_unsigned_to_nat(0u); x_46 = lean_nat_dec_eq(x_42, x_45); -x_14 = x_41; +x_14 = x_43; x_15 = x_42; -x_16 = x_43; +x_16 = x_41; x_17 = x_46; goto block_40; } @@ -41384,13 +41384,13 @@ lean_closure_set(x_46, 0, x_38); lean_closure_set(x_46, 1, x_28); lean_closure_set(x_46, 2, x_42); lean_closure_set(x_46, 3, x_4); -lean_closure_set(x_46, 4, x_26); +lean_closure_set(x_46, 4, x_27); lean_closure_set(x_46, 5, x_9); lean_closure_set(x_46, 6, x_10); lean_closure_set(x_46, 7, x_11); lean_closure_set(x_46, 8, x_18); lean_closure_set(x_46, 9, x_43); -lean_closure_set(x_46, 10, x_27); +lean_closure_set(x_46, 10, x_26); lean_closure_set(x_46, 11, x_17); lean_closure_set(x_46, 12, x_44); lean_closure_set(x_46, 13, x_14); @@ -41550,8 +41550,8 @@ if (x_79 == 0) lean_free_object(x_76); lean_free_object(x_67); lean_inc(x_69); -x_26 = x_69; -x_27 = x_64; +x_26 = x_64; +x_27 = x_69; x_28 = x_75; x_29 = x_69; x_30 = x_70; @@ -41581,8 +41581,8 @@ if (lean_obj_tag(x_83) == 0) { lean_dec_ref(x_83); lean_inc(x_69); -x_26 = x_69; -x_27 = x_64; +x_26 = x_64; +x_27 = x_69; x_28 = x_75; x_29 = x_69; x_30 = x_70; @@ -41646,8 +41646,8 @@ if (x_88 == 0) { lean_free_object(x_67); lean_inc(x_69); -x_26 = x_69; -x_27 = x_64; +x_26 = x_64; +x_27 = x_69; x_28 = x_75; x_29 = x_69; x_30 = x_70; @@ -41677,8 +41677,8 @@ if (lean_obj_tag(x_93) == 0) { lean_dec_ref(x_93); lean_inc(x_69); -x_26 = x_69; -x_27 = x_64; +x_26 = x_64; +x_27 = x_69; x_28 = x_75; x_29 = x_69; x_30 = x_70; @@ -41858,8 +41858,8 @@ if (x_113 == 0) { lean_dec(x_112); lean_inc(x_103); -x_26 = x_103; -x_27 = x_64; +x_26 = x_64; +x_27 = x_103; x_28 = x_109; x_29 = x_103; x_30 = x_104; @@ -41894,8 +41894,8 @@ if (lean_obj_tag(x_119) == 0) { lean_dec_ref(x_119); lean_inc(x_103); -x_26 = x_103; -x_27 = x_64; +x_26 = x_64; +x_27 = x_103; x_28 = x_109; x_29 = x_103; x_30 = x_104; @@ -47390,7 +47390,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_logErrorAt___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_checkNoInductiveNameConflicts_spec__0_spec__0___redArg(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) { _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; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -47425,15 +47425,15 @@ lean_ctor_set(x_25, 0, x_21); lean_ctor_set(x_25, 1, x_22); x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_13); +lean_ctor_set(x_26, 1, x_10); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_11); -lean_ctor_set(x_27, 1, x_10); -lean_ctor_set(x_27, 2, x_12); -lean_ctor_set(x_27, 3, x_14); +lean_ctor_set(x_27, 0, x_12); +lean_ctor_set(x_27, 1, x_15); +lean_ctor_set(x_27, 2, x_16); +lean_ctor_set(x_27, 3, x_13); lean_ctor_set(x_27, 4, x_26); -lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_16); -lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_15); +lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_11); +lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_14); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); lean_ctor_set(x_20, 6, x_28); @@ -47470,15 +47470,15 @@ lean_ctor_set(x_41, 0, x_21); lean_ctor_set(x_41, 1, x_22); x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_13); +lean_ctor_set(x_42, 1, x_10); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_11); -lean_ctor_set(x_43, 1, x_10); -lean_ctor_set(x_43, 2, x_12); -lean_ctor_set(x_43, 3, x_14); +lean_ctor_set(x_43, 0, x_12); +lean_ctor_set(x_43, 1, x_15); +lean_ctor_set(x_43, 2, x_16); +lean_ctor_set(x_43, 3, x_13); lean_ctor_set(x_43, 4, x_42); -lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_16); -lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_15); +lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_11); +lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_14); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); x_45 = lean_alloc_ctor(0, 9, 0); @@ -47508,10 +47508,10 @@ if (x_60 == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); -lean_inc_ref(x_56); -x_62 = l_Lean_FileMap_toPosition(x_56, x_53); -lean_dec(x_53); -x_63 = l_Lean_FileMap_toPosition(x_56, x_57); +lean_inc_ref(x_52); +x_62 = l_Lean_FileMap_toPosition(x_52, x_56); +lean_dec(x_56); +x_63 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); @@ -47520,13 +47520,13 @@ if (x_51 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); -x_10 = x_62; -x_11 = x_52; -x_12 = x_64; -x_13 = x_61; -x_14 = x_65; -x_15 = x_54; -x_16 = x_55; +x_10 = x_61; +x_11 = x_54; +x_12 = x_53; +x_13 = x_65; +x_14 = x_55; +x_15 = x_62; +x_16 = x_64; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -47543,7 +47543,7 @@ lean_object* x_67; lean_dec_ref(x_64); lean_dec_ref(x_62); lean_dec(x_61); -lean_dec_ref(x_52); +lean_dec_ref(x_53); lean_dec_ref(x_7); x_67 = lean_box(0); lean_ctor_set(x_59, 0, x_67); @@ -47552,13 +47552,13 @@ return x_59; else { lean_free_object(x_59); -x_10 = x_62; -x_11 = x_52; -x_12 = x_64; -x_13 = x_61; -x_14 = x_65; -x_15 = x_54; -x_16 = x_55; +x_10 = x_61; +x_11 = x_54; +x_12 = x_53; +x_13 = x_65; +x_14 = x_55; +x_15 = x_62; +x_16 = x_64; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -47572,10 +47572,10 @@ lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); -lean_inc_ref(x_56); -x_69 = l_Lean_FileMap_toPosition(x_56, x_53); -lean_dec(x_53); -x_70 = l_Lean_FileMap_toPosition(x_56, x_57); +lean_inc_ref(x_52); +x_69 = l_Lean_FileMap_toPosition(x_52, x_56); +lean_dec(x_56); +x_70 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); @@ -47583,13 +47583,13 @@ x_72 = l_Lean_addTrace___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab if (x_51 == 0) { lean_dec_ref(x_50); -x_10 = x_69; -x_11 = x_52; -x_12 = x_71; -x_13 = x_68; -x_14 = x_72; -x_15 = x_54; -x_16 = x_55; +x_10 = x_68; +x_11 = x_54; +x_12 = x_53; +x_13 = x_72; +x_14 = x_55; +x_15 = x_69; +x_16 = x_71; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -47606,7 +47606,7 @@ lean_object* x_74; lean_object* x_75; lean_dec_ref(x_71); lean_dec_ref(x_69); lean_dec(x_68); -lean_dec_ref(x_52); +lean_dec_ref(x_53); lean_dec_ref(x_7); x_74 = lean_box(0); x_75 = lean_alloc_ctor(0, 1, 0); @@ -47615,13 +47615,13 @@ return x_75; } else { -x_10 = x_69; -x_11 = x_52; -x_12 = x_71; -x_13 = x_68; -x_14 = x_72; -x_15 = x_54; -x_16 = x_55; +x_10 = x_68; +x_11 = x_54; +x_12 = x_53; +x_13 = x_72; +x_14 = x_55; +x_15 = x_69; +x_16 = x_71; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -47633,7 +47633,7 @@ goto block_49; block_87: { lean_object* x_85; -x_85 = l_Lean_Syntax_getTailPos_x3f(x_80, x_82); +x_85 = l_Lean_Syntax_getTailPos_x3f(x_80, x_81); lean_dec(x_80); if (lean_obj_tag(x_85) == 0) { @@ -47641,10 +47641,10 @@ lean_inc(x_84); x_50 = x_77; x_51 = x_78; x_52 = x_79; -x_53 = x_84; +x_53 = x_82; x_54 = x_81; -x_55 = x_82; -x_56 = x_83; +x_55 = x_83; +x_56 = x_84; x_57 = x_84; goto block_76; } @@ -47657,10 +47657,10 @@ lean_dec_ref(x_85); x_50 = x_77; x_51 = x_78; x_52 = x_79; -x_53 = x_84; +x_53 = x_82; x_54 = x_81; -x_55 = x_82; -x_56 = x_83; +x_55 = x_83; +x_56 = x_84; x_57 = x_86; goto block_76; } @@ -47668,8 +47668,8 @@ goto block_76; block_99: { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_replaceRef(x_1, x_91); -lean_dec(x_91); +x_95 = l_Lean_replaceRef(x_1, x_93); +lean_dec(x_93); x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_92); if (lean_obj_tag(x_96) == 0) { @@ -47679,9 +47679,9 @@ x_77 = x_88; x_78 = x_89; x_79 = x_90; x_80 = x_95; -x_81 = x_94; -x_82 = x_92; -x_83 = x_93; +x_81 = x_92; +x_82 = x_91; +x_83 = x_94; x_84 = x_97; goto block_87; } @@ -47695,9 +47695,9 @@ x_77 = x_88; x_78 = x_89; x_79 = x_90; x_80 = x_95; -x_81 = x_94; -x_82 = x_92; -x_83 = x_93; +x_81 = x_92; +x_82 = x_91; +x_83 = x_94; x_84 = x_98; goto block_87; } @@ -47706,10 +47706,10 @@ goto block_87; { if (x_107 == 0) { -x_88 = x_104; +x_88 = x_103; x_89 = x_101; x_90 = x_102; -x_91 = x_103; +x_91 = x_104; x_92 = x_106; x_93 = x_105; x_94 = x_3; @@ -47717,10 +47717,10 @@ goto block_99; } else { -x_88 = x_104; +x_88 = x_103; x_89 = x_101; x_90 = x_102; -x_91 = x_103; +x_91 = x_104; x_92 = x_106; x_93 = x_105; x_94 = x_100; @@ -47746,14 +47746,14 @@ x_118 = 1; x_119 = l_Lean_instBEqMessageSeverity_beq(x_3, x_118); if (x_119 == 0) { -lean_inc_ref(x_111); lean_inc(x_113); lean_inc_ref(x_110); +lean_inc_ref(x_111); x_101 = x_114; -x_102 = x_110; -x_103 = x_113; -x_104 = x_117; -x_105 = x_111; +x_102 = x_111; +x_103 = x_117; +x_104 = x_110; +x_105 = x_113; x_106 = x_109; x_107 = x_119; goto block_108; @@ -47763,14 +47763,14 @@ else lean_object* x_120; uint8_t x_121; x_120 = l_Lean_logAt___at___00Lean_logErrorAt___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_checkNoInductiveNameConflicts_spec__0_spec__0___redArg___closed__0; x_121 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_throwErrorAt___at___00Lean_Elab_Command_mkInductiveView_spec__0_spec__0_spec__2_spec__3(x_112, x_120); -lean_inc_ref(x_111); lean_inc(x_113); lean_inc_ref(x_110); +lean_inc_ref(x_111); x_101 = x_114; -x_102 = x_110; -x_103 = x_113; -x_104 = x_117; -x_105 = x_111; +x_102 = x_111; +x_103 = x_117; +x_104 = x_110; +x_105 = x_113; x_106 = x_109; x_107 = x_121; goto block_108; @@ -49697,7 +49697,7 @@ return x_7; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__2_spec__2_spec__3(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_8; lean_object* x_9; uint8_t 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; uint8_t x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; uint8_t x_116; lean_object* x_117; uint8_t x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; uint8_t x_125; uint8_t x_126; lean_object* x_127; uint8_t x_128; uint8_t x_139; uint8_t x_140; uint8_t x_141; lean_object* x_142; uint8_t x_143; uint8_t x_145; uint8_t x_158; +lean_object* x_8; uint8_t 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; uint8_t x_82; uint8_t x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; uint8_t x_116; uint8_t x_117; lean_object* x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; uint8_t x_125; lean_object* x_126; uint8_t x_127; uint8_t x_128; uint8_t x_139; uint8_t x_140; lean_object* x_141; uint8_t x_142; uint8_t x_143; uint8_t x_145; uint8_t x_158; x_139 = 2; x_158 = l_Lean_instBEqMessageSeverity_beq(x_3, x_139); if (x_158 == 0) @@ -49749,15 +49749,15 @@ lean_ctor_set(x_27, 0, x_23); lean_ctor_set(x_27, 1, x_24); x_28 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_9); +lean_ctor_set(x_28, 1, x_13); x_29 = lean_alloc_ctor(0, 5, 3); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_12); -lean_ctor_set(x_29, 2, x_8); -lean_ctor_set(x_29, 3, x_13); +lean_ctor_set(x_29, 2, x_10); +lean_ctor_set(x_29, 3, x_8); lean_ctor_set(x_29, 4, x_28); -lean_ctor_set_uint8(x_29, sizeof(void*)*5, x_10); -lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 1, x_14); +lean_ctor_set_uint8(x_29, sizeof(void*)*5, x_14); +lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 1, x_9); lean_ctor_set_uint8(x_29, sizeof(void*)*5 + 2, x_4); x_30 = l_Lean_MessageLog_add(x_29, x_26); lean_ctor_set(x_22, 1, x_30); @@ -49797,15 +49797,15 @@ lean_ctor_set(x_44, 0, x_23); lean_ctor_set(x_44, 1, x_24); x_45 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_9); +lean_ctor_set(x_45, 1, x_13); x_46 = lean_alloc_ctor(0, 5, 3); lean_ctor_set(x_46, 0, x_11); lean_ctor_set(x_46, 1, x_12); -lean_ctor_set(x_46, 2, x_8); -lean_ctor_set(x_46, 3, x_13); +lean_ctor_set(x_46, 2, x_10); +lean_ctor_set(x_46, 3, x_8); lean_ctor_set(x_46, 4, x_45); -lean_ctor_set_uint8(x_46, sizeof(void*)*5, x_10); -lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 1, x_14); +lean_ctor_set_uint8(x_46, sizeof(void*)*5, x_14); +lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 1, x_9); lean_ctor_set_uint8(x_46, sizeof(void*)*5 + 2, x_4); x_47 = l_Lean_MessageLog_add(x_46, x_34); x_48 = lean_alloc_ctor(0, 11, 0); @@ -49883,15 +49883,15 @@ lean_ctor_set(x_67, 0, x_53); lean_ctor_set(x_67, 1, x_54); x_68 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_9); +lean_ctor_set(x_68, 1, x_13); x_69 = lean_alloc_ctor(0, 5, 3); lean_ctor_set(x_69, 0, x_11); lean_ctor_set(x_69, 1, x_12); -lean_ctor_set(x_69, 2, x_8); -lean_ctor_set(x_69, 3, x_13); +lean_ctor_set(x_69, 2, x_10); +lean_ctor_set(x_69, 3, x_8); lean_ctor_set(x_69, 4, x_68); -lean_ctor_set_uint8(x_69, sizeof(void*)*5, x_10); -lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 1, x_14); +lean_ctor_set_uint8(x_69, sizeof(void*)*5, x_14); +lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 1, x_9); lean_ctor_set_uint8(x_69, sizeof(void*)*5 + 2, x_4); x_70 = l_Lean_MessageLog_add(x_69, x_56); if (lean_is_scalar(x_66)) { @@ -49924,8 +49924,8 @@ lean_dec(x_18); lean_dec_ref(x_13); lean_dec_ref(x_12); lean_dec_ref(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_10); +lean_dec_ref(x_8); x_75 = !lean_is_exclusive(x_19); if (x_75 == 0) { @@ -49949,8 +49949,8 @@ uint8_t x_78; lean_dec_ref(x_13); lean_dec_ref(x_12); lean_dec_ref(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_10); +lean_dec_ref(x_8); x_78 = !lean_is_exclusive(x_17); if (x_78 == 0) { @@ -49995,12 +49995,12 @@ x_98 = l_Lean_addTrace___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab if (x_90 == 0) { lean_free_object(x_92); -x_8 = x_97; -x_9 = x_94; -x_10 = x_84; +x_8 = x_98; +x_9 = x_83; +x_10 = x_97; x_11 = x_88; x_12 = x_95; -x_13 = x_98; +x_13 = x_94; x_14 = x_86; x_15 = x_6; x_16 = lean_box(0); @@ -50030,12 +50030,12 @@ return x_92; else { lean_free_object(x_92); -x_8 = x_97; -x_9 = x_94; -x_10 = x_84; +x_8 = x_98; +x_9 = x_83; +x_10 = x_97; x_11 = x_88; x_12 = x_95; -x_13 = x_98; +x_13 = x_94; x_14 = x_86; x_15 = x_6; x_16 = lean_box(0); @@ -50059,12 +50059,12 @@ lean_ctor_set(x_107, 0, x_106); x_108 = l_Lean_addTrace___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux_spec__3___redArg___closed__1; if (x_90 == 0) { -x_8 = x_107; -x_9 = x_104; -x_10 = x_84; +x_8 = x_108; +x_9 = x_83; +x_10 = x_107; x_11 = x_88; x_12 = x_105; -x_13 = x_108; +x_13 = x_104; x_14 = x_86; x_15 = x_6; x_16 = lean_box(0); @@ -50094,12 +50094,12 @@ return x_114; } else { -x_8 = x_107; -x_9 = x_104; -x_10 = x_84; +x_8 = x_108; +x_9 = x_83; +x_10 = x_107; x_11 = x_88; x_12 = x_105; -x_13 = x_108; +x_13 = x_104; x_14 = x_86; x_15 = x_6; x_16 = lean_box(0); @@ -50111,14 +50111,14 @@ goto block_81; block_124: { lean_object* x_122; -x_122 = l_Lean_Syntax_getTailPos_x3f(x_119, x_118); +x_122 = l_Lean_Syntax_getTailPos_x3f(x_119, x_120); lean_dec(x_119); if (lean_obj_tag(x_122) == 0) { lean_inc(x_121); x_82 = x_116; -x_83 = lean_box(0); -x_84 = x_118; +x_83 = x_117; +x_84 = lean_box(0); x_85 = x_121; x_86 = x_120; x_87 = x_121; @@ -50131,8 +50131,8 @@ x_123 = lean_ctor_get(x_122, 0); lean_inc(x_123); lean_dec_ref(x_122); x_82 = x_116; -x_83 = lean_box(0); -x_84 = x_118; +x_83 = x_117; +x_84 = lean_box(0); x_85 = x_121; x_86 = x_120; x_87 = x_123; @@ -50151,16 +50151,16 @@ lean_inc(x_130); lean_dec_ref(x_129); x_131 = l_Lean_replaceRef(x_1, x_130); lean_dec(x_130); -x_132 = l_Lean_Syntax_getPos_x3f(x_131, x_126); +x_132 = l_Lean_Syntax_getPos_x3f(x_131, x_127); if (lean_obj_tag(x_132) == 0) { lean_object* x_133; x_133 = lean_unsigned_to_nat(0u); x_116 = x_125; -x_117 = lean_box(0); -x_118 = x_126; +x_117 = x_128; +x_118 = lean_box(0); x_119 = x_131; -x_120 = x_128; +x_120 = x_127; x_121 = x_133; goto block_124; } @@ -50171,10 +50171,10 @@ x_134 = lean_ctor_get(x_132, 0); lean_inc(x_134); lean_dec_ref(x_132); x_116 = x_125; -x_117 = lean_box(0); -x_118 = x_126; +x_117 = x_128; +x_118 = lean_box(0); x_119 = x_131; -x_120 = x_128; +x_120 = x_127; x_121 = x_134; goto block_124; } @@ -50206,16 +50206,16 @@ return x_137; if (x_143 == 0) { x_125 = x_140; -x_126 = x_141; -x_127 = lean_box(0); +x_126 = lean_box(0); +x_127 = x_142; x_128 = x_3; goto block_138; } else { x_125 = x_140; -x_126 = x_141; -x_127 = lean_box(0); +x_126 = lean_box(0); +x_127 = x_142; x_128 = x_139; goto block_138; } @@ -50241,8 +50241,8 @@ if (x_152 == 0) { lean_dec(x_150); x_140 = x_145; -x_141 = x_145; -x_142 = lean_box(0); +x_141 = lean_box(0); +x_142 = x_145; x_143 = x_152; goto block_144; } @@ -50253,8 +50253,8 @@ x_153 = l_Lean_logAt___at___00Lean_logErrorAt___at___00__private_Lean_Elab_Mutua x_154 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_throwErrorAt___at___00Lean_Elab_Command_mkInductiveView_spec__0_spec__0_spec__2_spec__3(x_150, x_153); lean_dec(x_150); x_140 = x_145; -x_141 = x_145; -x_142 = lean_box(0); +x_141 = lean_box(0); +x_142 = x_145; x_143 = x_154; goto block_144; } @@ -51543,24 +51543,24 @@ goto block_528; 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 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux___lam__1___closed__15; x_19 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__0___closed__9; -lean_inc(x_15); +lean_inc(x_16); x_20 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 0, x_16); lean_ctor_set(x_20, 1, x_18); lean_ctor_set(x_20, 2, x_19); x_21 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___closed__5; x_22 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_21); -lean_inc(x_15); +lean_inc(x_16); x_23 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_23, 0, x_15); +lean_ctor_set(x_23, 0, x_16); lean_ctor_set(x_23, 1, x_21); -lean_inc(x_15); -x_24 = l_Lean_Syntax_node1(x_15, x_22, x_23); -lean_inc(x_15); -x_25 = l_Lean_Syntax_node1(x_15, x_18, x_24); +lean_inc(x_16); +x_24 = l_Lean_Syntax_node1(x_16, x_22, x_23); +lean_inc(x_16); +x_25 = l_Lean_Syntax_node1(x_16, x_18, x_24); lean_inc_ref_n(x_20, 5); -x_26 = l_Lean_Syntax_node7(x_15, x_4, x_20, x_20, x_20, x_20, x_25, x_20, x_20); -x_27 = lean_apply_4(x_5, x_26, x_14, x_16, lean_box(0)); +x_26 = l_Lean_Syntax_node7(x_16, x_4, x_20, x_20, x_20, x_20, x_25, x_20, x_20); +x_27 = lean_apply_4(x_5, x_26, x_15, x_14, lean_box(0)); return x_27; } block_43: @@ -51585,60 +51585,60 @@ lean_inc(x_29); x_40 = l_Lean_Syntax_node1(x_29, x_33, x_39); lean_inc_ref_n(x_35, 5); x_41 = l_Lean_Syntax_node7(x_29, x_4, x_35, x_35, x_35, x_35, x_40, x_35, x_35); -x_42 = lean_apply_4(x_5, x_41, x_30, x_31, lean_box(0)); +x_42 = lean_apply_4(x_5, x_41, x_31, x_30, lean_box(0)); return x_42; } block_64: { 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_inc_ref(x_50); -x_54 = l_Array_append___redArg(x_50, x_53); +lean_inc_ref(x_44); +x_54 = l_Array_append___redArg(x_44, x_53); lean_dec_ref(x_53); -lean_inc(x_52); -lean_inc(x_46); +lean_inc(x_51); +lean_inc(x_45); x_55 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_55, 0, x_46); -lean_ctor_set(x_55, 1, x_52); +lean_ctor_set(x_55, 0, x_45); +lean_ctor_set(x_55, 1, x_51); lean_ctor_set(x_55, 2, x_54); x_56 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___closed__5; x_57 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_56); -lean_inc(x_46); +lean_inc(x_45); x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_46); +lean_ctor_set(x_58, 0, x_45); lean_ctor_set(x_58, 1, x_56); -lean_inc(x_46); -x_59 = l_Lean_Syntax_node1(x_46, x_57, x_58); -lean_inc(x_52); -lean_inc(x_46); -x_60 = l_Lean_Syntax_node1(x_46, x_52, x_59); -lean_inc(x_46); +lean_inc(x_45); +x_59 = l_Lean_Syntax_node1(x_45, x_57, x_58); +lean_inc(x_51); +lean_inc(x_45); +x_60 = l_Lean_Syntax_node1(x_45, x_51, x_59); +lean_inc(x_45); x_61 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_61, 0, x_46); -lean_ctor_set(x_61, 1, x_52); -lean_ctor_set(x_61, 2, x_50); +lean_ctor_set(x_61, 0, x_45); +lean_ctor_set(x_61, 1, x_51); +lean_ctor_set(x_61, 2, x_44); lean_inc_ref(x_61); -x_62 = l_Lean_Syntax_node7(x_46, x_4, x_51, x_48, x_45, x_55, x_60, x_61, x_61); -x_63 = lean_apply_4(x_5, x_62, x_44, x_49, lean_box(0)); +x_62 = l_Lean_Syntax_node7(x_45, x_4, x_50, x_47, x_46, x_55, x_60, x_61, x_61); +x_63 = lean_apply_4(x_5, x_62, x_52, x_49, lean_box(0)); return x_63; } block_85: { lean_object* x_75; lean_object* x_76; -lean_inc_ref(x_71); -x_75 = l_Array_append___redArg(x_71, x_74); +lean_inc_ref(x_65); +x_75 = l_Array_append___redArg(x_65, x_74); lean_dec_ref(x_74); -lean_inc(x_73); +lean_inc(x_72); lean_inc(x_66); x_76 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_76, 0, x_66); -lean_ctor_set(x_76, 1, x_73); +lean_ctor_set(x_76, 1, x_72); lean_ctor_set(x_76, 2, x_75); -if (lean_obj_tag(x_69) == 1) +if (lean_obj_tag(x_68) == 1) { lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_77 = lean_ctor_get(x_69, 0); +x_77 = lean_ctor_get(x_68, 0); lean_inc(x_77); -lean_dec_ref(x_69); +lean_dec_ref(x_68); x_78 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__1___closed__0; lean_inc_ref(x_3); lean_inc_ref(x_2); @@ -51653,12 +51653,12 @@ lean_inc(x_66); x_82 = l_Lean_Syntax_node1(x_66, x_79, x_81); x_83 = l_Array_mkArray1___redArg(x_82); x_44 = x_65; -x_45 = x_76; -x_46 = x_66; -x_47 = lean_box(0); -x_48 = x_68; -x_49 = x_70; -x_50 = x_71; +x_45 = x_66; +x_46 = x_76; +x_47 = x_67; +x_48 = lean_box(0); +x_49 = x_71; +x_50 = x_70; x_51 = x_72; x_52 = x_73; x_53 = x_83; @@ -51667,15 +51667,15 @@ goto block_64; else { lean_object* x_84; -lean_dec(x_69); +lean_dec(x_68); x_84 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__1___closed__1; x_44 = x_65; -x_45 = x_76; -x_46 = x_66; -x_47 = lean_box(0); -x_48 = x_68; -x_49 = x_70; -x_50 = x_71; +x_45 = x_66; +x_46 = x_76; +x_47 = x_67; +x_48 = lean_box(0); +x_49 = x_71; +x_50 = x_70; x_51 = x_72; x_52 = x_73; x_53 = x_84; @@ -51685,29 +51685,29 @@ goto block_64; block_101: { lean_object* x_96; lean_object* x_97; -lean_inc_ref(x_92); -x_96 = l_Array_append___redArg(x_92, x_95); +lean_inc_ref(x_86); +x_96 = l_Array_append___redArg(x_86, x_95); lean_dec_ref(x_95); -lean_inc(x_94); -lean_inc(x_88); +lean_inc(x_93); +lean_inc(x_87); x_97 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_97, 0, x_88); -lean_ctor_set(x_97, 1, x_94); +lean_ctor_set(x_97, 0, x_87); +lean_ctor_set(x_97, 1, x_93); lean_ctor_set(x_97, 2, x_96); -if (lean_obj_tag(x_86) == 1) +if (lean_obj_tag(x_90) == 1) { lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_86, 0); +x_98 = lean_ctor_get(x_90, 0); lean_inc(x_98); -lean_dec_ref(x_86); +lean_dec_ref(x_90); x_99 = l_Array_mkArray1___redArg(x_98); -x_65 = x_87; -x_66 = x_88; -x_67 = lean_box(0); -x_68 = x_97; -x_69 = x_90; -x_70 = x_91; -x_71 = x_92; +x_65 = x_86; +x_66 = x_87; +x_67 = x_97; +x_68 = x_88; +x_69 = lean_box(0); +x_70 = x_92; +x_71 = x_91; x_72 = x_93; x_73 = x_94; x_74 = x_99; @@ -51716,15 +51716,15 @@ goto block_85; else { lean_object* x_100; -lean_dec(x_86); +lean_dec(x_90); x_100 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__1___closed__1; -x_65 = x_87; -x_66 = x_88; -x_67 = lean_box(0); -x_68 = x_97; -x_69 = x_90; -x_70 = x_91; -x_71 = x_92; +x_65 = x_86; +x_66 = x_87; +x_67 = x_97; +x_68 = x_88; +x_69 = lean_box(0); +x_70 = x_92; +x_71 = x_91; x_72 = x_93; x_73 = x_94; x_74 = x_100; @@ -51734,30 +51734,30 @@ goto block_85; block_117: { lean_object* x_112; lean_object* x_113; -lean_inc_ref(x_109); -x_112 = l_Array_append___redArg(x_109, x_111); +lean_inc_ref(x_102); +x_112 = l_Array_append___redArg(x_102, x_111); lean_dec_ref(x_111); -lean_inc(x_110); -lean_inc(x_105); +lean_inc(x_109); +lean_inc(x_104); x_113 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_113, 0, x_105); -lean_ctor_set(x_113, 1, x_110); +lean_ctor_set(x_113, 0, x_104); +lean_ctor_set(x_113, 1, x_109); lean_ctor_set(x_113, 2, x_112); -if (lean_obj_tag(x_102) == 1) +if (lean_obj_tag(x_103) == 1) { lean_object* x_114; lean_object* x_115; -x_114 = lean_ctor_get(x_102, 0); +x_114 = lean_ctor_get(x_103, 0); lean_inc(x_114); -lean_dec_ref(x_102); +lean_dec_ref(x_103); x_115 = l_Array_mkArray1___redArg(x_114); -x_86 = x_104; -x_87 = x_103; +x_86 = x_102; +x_87 = x_104; x_88 = x_105; x_89 = lean_box(0); x_90 = x_107; x_91 = x_108; -x_92 = x_109; -x_93 = x_113; +x_92 = x_113; +x_93 = x_109; x_94 = x_110; x_95 = x_115; goto block_101; @@ -51765,16 +51765,16 @@ goto block_101; else { lean_object* x_116; -lean_dec(x_102); +lean_dec(x_103); x_116 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__1___closed__1; -x_86 = x_104; -x_87 = x_103; +x_86 = x_102; +x_87 = x_104; x_88 = x_105; x_89 = lean_box(0); x_90 = x_107; x_91 = x_108; -x_92 = x_109; -x_93 = x_113; +x_92 = x_113; +x_93 = x_109; x_94 = x_110; x_95 = x_116; goto block_101; @@ -51792,15 +51792,15 @@ x_127 = lean_ctor_get(x_10, 0); lean_inc(x_127); lean_dec_ref(x_10); x_128 = l_Array_mkArray1___redArg(x_127); -x_102 = x_118; -x_103 = x_121; -x_104 = x_120; -x_105 = x_119; +x_102 = x_126; +x_103 = x_119; +x_104 = x_118; +x_105 = x_120; x_106 = lean_box(0); -x_107 = x_122; -x_108 = x_123; -x_109 = x_126; -x_110 = x_125; +x_107 = x_121; +x_108 = x_122; +x_109 = x_125; +x_110 = x_123; x_111 = x_128; goto block_117; } @@ -51809,15 +51809,15 @@ else lean_object* x_129; lean_dec(x_10); x_129 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__1___closed__1; -x_102 = x_118; -x_103 = x_121; -x_104 = x_120; -x_105 = x_119; +x_102 = x_126; +x_103 = x_119; +x_104 = x_118; +x_105 = x_120; x_106 = lean_box(0); -x_107 = x_122; -x_108 = x_123; -x_109 = x_126; -x_110 = x_125; +x_107 = x_121; +x_108 = x_122; +x_109 = x_125; +x_110 = x_123; x_111 = x_129; goto block_117; } @@ -51902,9 +51902,9 @@ x_160 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_160) == 0) { lean_dec_ref(x_160); -x_14 = x_134; -x_15 = x_159; -x_16 = x_135; +x_14 = x_135; +x_15 = x_134; +x_16 = x_159; x_17 = lean_box(0); goto block_28; } @@ -51938,9 +51938,9 @@ return x_163; } else { -x_14 = x_134; -x_15 = x_159; -x_16 = x_135; +x_14 = x_135; +x_15 = x_134; +x_16 = x_159; x_17 = lean_box(0); goto block_28; } @@ -52135,8 +52135,8 @@ if (lean_obj_tag(x_199) == 0) { lean_dec_ref(x_199); x_29 = x_198; -x_30 = x_134; -x_31 = x_135; +x_30 = x_135; +x_31 = x_134; x_32 = lean_box(0); goto block_43; } @@ -52171,8 +52171,8 @@ return x_202; else { x_29 = x_198; -x_30 = x_134; -x_31 = x_135; +x_30 = x_135; +x_31 = x_134; x_32 = lean_box(0); goto block_43; } @@ -52312,12 +52312,12 @@ x_221 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_221) == 0) { lean_dec_ref(x_221); -x_118 = x_131; -x_119 = x_220; +x_118 = x_220; +x_119 = x_131; x_120 = x_132; -x_121 = x_134; -x_122 = x_133; -x_123 = x_135; +x_121 = x_133; +x_122 = x_135; +x_123 = x_134; x_124 = lean_box(0); goto block_130; } @@ -52355,12 +52355,12 @@ return x_224; } else { -x_118 = x_131; -x_119 = x_220; +x_118 = x_220; +x_119 = x_131; x_120 = x_132; -x_121 = x_134; -x_122 = x_133; -x_123 = x_135; +x_121 = x_133; +x_122 = x_135; +x_123 = x_134; x_124 = lean_box(0); goto block_130; } @@ -52435,24 +52435,24 @@ return x_230; 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_236 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux___lam__1___closed__15; x_237 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__0___closed__9; -lean_inc(x_233); +lean_inc(x_234); x_238 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_238, 0, x_233); +lean_ctor_set(x_238, 0, x_234); lean_ctor_set(x_238, 1, x_236); lean_ctor_set(x_238, 2, x_237); x_239 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___closed__5; x_240 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_239); -lean_inc(x_233); +lean_inc(x_234); x_241 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_241, 0, x_233); +lean_ctor_set(x_241, 0, x_234); lean_ctor_set(x_241, 1, x_239); -lean_inc(x_233); -x_242 = l_Lean_Syntax_node1(x_233, x_240, x_241); -lean_inc(x_233); -x_243 = l_Lean_Syntax_node1(x_233, x_236, x_242); +lean_inc(x_234); +x_242 = l_Lean_Syntax_node1(x_234, x_240, x_241); +lean_inc(x_234); +x_243 = l_Lean_Syntax_node1(x_234, x_236, x_242); lean_inc_ref_n(x_238, 5); -x_244 = l_Lean_Syntax_node7(x_233, x_4, x_238, x_238, x_238, x_238, x_243, x_238, x_238); -x_245 = lean_apply_4(x_5, x_244, x_232, x_234, lean_box(0)); +x_244 = l_Lean_Syntax_node7(x_234, x_4, x_238, x_238, x_238, x_238, x_243, x_238, x_238); +x_245 = lean_apply_4(x_5, x_244, x_233, x_232, lean_box(0)); return x_245; } block_261: @@ -52460,22 +52460,22 @@ return x_245; 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; x_253 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux___lam__1___closed__15; x_254 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__0___closed__9; -lean_inc(x_250); +lean_inc(x_251); x_255 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_255, 0, x_250); +lean_ctor_set(x_255, 0, x_251); lean_ctor_set(x_255, 1, x_253); lean_ctor_set(x_255, 2, x_254); -lean_inc(x_250); +lean_inc(x_251); x_256 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_256, 0, x_250); -lean_ctor_set(x_256, 1, x_247); -lean_inc(x_250); -x_257 = l_Lean_Syntax_node1(x_250, x_248, x_256); -lean_inc(x_250); -x_258 = l_Lean_Syntax_node1(x_250, x_253, x_257); +lean_ctor_set(x_256, 0, x_251); +lean_ctor_set(x_256, 1, x_250); +lean_inc(x_251); +x_257 = l_Lean_Syntax_node1(x_251, x_248, x_256); +lean_inc(x_251); +x_258 = l_Lean_Syntax_node1(x_251, x_253, x_257); lean_inc_ref_n(x_255, 5); -x_259 = l_Lean_Syntax_node7(x_250, x_4, x_255, x_255, x_255, x_255, x_258, x_255, x_255); -x_260 = lean_apply_4(x_5, x_259, x_249, x_251, lean_box(0)); +x_259 = l_Lean_Syntax_node7(x_251, x_4, x_255, x_255, x_255, x_255, x_258, x_255, x_255); +x_260 = lean_apply_4(x_5, x_259, x_249, x_247, lean_box(0)); return x_260; } block_276: @@ -52483,24 +52483,24 @@ return x_260; 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; x_266 = l___private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_elabHeadersAux___lam__1___closed__15; x_267 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___lam__0___closed__9; -lean_inc(x_264); +lean_inc(x_263); x_268 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_268, 0, x_264); +lean_ctor_set(x_268, 0, x_263); lean_ctor_set(x_268, 1, x_266); lean_ctor_set(x_268, 2, x_267); x_269 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_MutualInductive_0__Lean_Elab_Command_applyComputedFields_spec__3___closed__5; x_270 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_269); -lean_inc(x_264); +lean_inc(x_263); x_271 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_271, 0, x_264); +lean_ctor_set(x_271, 0, x_263); lean_ctor_set(x_271, 1, x_269); -lean_inc(x_264); -x_272 = l_Lean_Syntax_node1(x_264, x_270, x_271); -lean_inc(x_264); -x_273 = l_Lean_Syntax_node1(x_264, x_266, x_272); +lean_inc(x_263); +x_272 = l_Lean_Syntax_node1(x_263, x_270, x_271); +lean_inc(x_263); +x_273 = l_Lean_Syntax_node1(x_263, x_266, x_272); lean_inc_ref_n(x_268, 5); -x_274 = l_Lean_Syntax_node7(x_264, x_4, x_268, x_268, x_268, x_268, x_273, x_268, x_268); -x_275 = lean_apply_4(x_5, x_274, x_263, x_262, lean_box(0)); +x_274 = l_Lean_Syntax_node7(x_263, x_4, x_268, x_268, x_268, x_268, x_273, x_268, x_268); +x_275 = lean_apply_4(x_5, x_274, x_262, x_264, lean_box(0)); return x_275; } block_291: @@ -52525,7 +52525,7 @@ lean_inc(x_279); x_288 = l_Lean_Syntax_node1(x_279, x_281, x_287); lean_inc_ref_n(x_283, 5); x_289 = l_Lean_Syntax_node7(x_279, x_4, x_283, x_283, x_283, x_283, x_288, x_283, x_283); -x_290 = lean_apply_4(x_5, x_289, x_278, x_277, lean_box(0)); +x_290 = lean_apply_4(x_5, x_289, x_277, x_278, lean_box(0)); return x_290; } block_306: @@ -52550,7 +52550,7 @@ lean_inc(x_293); x_303 = l_Lean_Syntax_node1(x_293, x_296, x_302); lean_inc_ref_n(x_298, 5); x_304 = l_Lean_Syntax_node7(x_293, x_4, x_298, x_298, x_298, x_298, x_303, x_298, x_298); -x_305 = lean_apply_4(x_5, x_304, x_292, x_294, lean_box(0)); +x_305 = lean_apply_4(x_5, x_304, x_294, x_292, lean_box(0)); return x_305; } block_394: @@ -52639,9 +52639,9 @@ x_338 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_338) == 0) { lean_dec_ref(x_338); -x_232 = x_311; -x_233 = x_337; -x_234 = x_312; +x_232 = x_312; +x_233 = x_311; +x_234 = x_337; x_235 = lean_box(0); goto block_246; } @@ -52675,9 +52675,9 @@ return x_341; } else { -x_232 = x_311; -x_233 = x_337; -x_234 = x_312; +x_232 = x_312; +x_233 = x_311; +x_234 = x_337; x_235 = lean_box(0); goto block_246; } @@ -52879,11 +52879,11 @@ x_378 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_378) == 0) { lean_dec_ref(x_378); -x_247 = x_355; +x_247 = x_312; x_248 = x_356; x_249 = x_311; -x_250 = x_377; -x_251 = x_312; +x_250 = x_355; +x_251 = x_377; x_252 = lean_box(0); goto block_261; } @@ -52915,11 +52915,11 @@ return x_381; } else { -x_247 = x_355; +x_247 = x_312; x_248 = x_356; x_249 = x_311; -x_250 = x_377; -x_251 = x_312; +x_250 = x_355; +x_251 = x_377; x_252 = lean_box(0); goto block_261; } @@ -53029,8 +53029,8 @@ else { lean_dec(x_356); x_131 = x_308; -x_132 = x_309; -x_133 = x_310; +x_132 = x_310; +x_133 = x_309; x_134 = x_311; x_135 = x_312; x_136 = lean_box(0); @@ -53042,8 +53042,8 @@ else { lean_dec(x_315); x_131 = x_308; -x_132 = x_309; -x_133 = x_310; +x_132 = x_310; +x_133 = x_309; x_134 = x_311; x_135 = x_312; x_136 = lean_box(0); @@ -53135,9 +53135,9 @@ x_424 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_424) == 0) { lean_dec_ref(x_424); -x_262 = x_398; -x_263 = x_397; -x_264 = x_423; +x_262 = x_397; +x_263 = x_423; +x_264 = x_398; x_265 = lean_box(0); goto block_276; } @@ -53171,9 +53171,9 @@ return x_427; } else { -x_262 = x_398; -x_263 = x_397; -x_264 = x_423; +x_262 = x_397; +x_263 = x_423; +x_264 = x_398; x_265 = lean_box(0); goto block_276; } @@ -53374,8 +53374,8 @@ x_464 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_464) == 0) { lean_dec_ref(x_464); -x_277 = x_398; -x_278 = x_397; +x_277 = x_397; +x_278 = x_398; x_279 = x_463; x_280 = lean_box(0); goto block_291; @@ -53410,8 +53410,8 @@ return x_467; } else { -x_277 = x_398; -x_278 = x_397; +x_277 = x_397; +x_278 = x_398; x_279 = x_463; x_280 = lean_box(0); goto block_291; @@ -53641,9 +53641,9 @@ x_509 = l_Lean_getMainModule___at___00__private_Lean_Elab_MutualInductive_0__Lea if (lean_obj_tag(x_509) == 0) { lean_dec_ref(x_509); -x_292 = x_11; +x_292 = x_12; x_293 = x_508; -x_294 = x_12; +x_294 = x_11; x_295 = lean_box(0); goto block_306; } @@ -53677,9 +53677,9 @@ return x_512; } else { -x_292 = x_11; +x_292 = x_12; x_293 = x_508; -x_294 = x_12; +x_294 = x_11; x_295 = lean_box(0); goto block_306; } @@ -62122,7 +62122,7 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___00Lean_Elab_Command_elabMutualInductive_spec__0(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; uint8_t x_16; lean_object* 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; uint8_t x_40; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_86; lean_object* x_87; uint8_t x_88; uint8_t x_109; lean_object* x_123; lean_object* x_124; uint8_t x_125; +uint8_t x_5; uint8_t x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; uint8_t x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_86; lean_object* x_87; uint8_t x_88; uint8_t x_109; lean_object* x_123; lean_object* x_124; uint8_t x_125; x_28 = lean_unsigned_to_nat(0u); x_29 = l_Lean_Syntax_getArg(x_1, x_28); x_30 = lean_unsigned_to_nat(1u); @@ -62171,11 +62171,11 @@ goto block_122; lean_object* x_13; lean_object* x_14; x_13 = lean_alloc_ctor(0, 3, 5); lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_6); -lean_ctor_set(x_13, 2, x_8); -lean_ctor_set_uint8(x_13, sizeof(void*)*3, x_9); +lean_ctor_set(x_13, 1, x_10); +lean_ctor_set(x_13, 2, x_9); +lean_ctor_set_uint8(x_13, sizeof(void*)*3, x_6); lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 1, x_11); -lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 2, x_8); lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 3, x_5); lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 4, x_12); x_14 = lean_alloc_ctor(0, 1, 0); @@ -62185,19 +62185,19 @@ return x_14; block_27: { uint8_t x_24; -x_24 = l_Lean_Syntax_isNone(x_21); -lean_dec(x_21); +x_24 = l_Lean_Syntax_isNone(x_19); +lean_dec(x_19); if (x_24 == 0) { uint8_t x_25; x_25 = 1; -x_5 = x_16; -x_6 = x_17; -x_7 = x_18; -x_8 = x_22; -x_9 = x_19; -x_10 = lean_box(0); -x_11 = x_20; +x_5 = x_17; +x_6 = x_16; +x_7 = lean_box(0); +x_8 = x_18; +x_9 = x_22; +x_10 = x_20; +x_11 = x_21; x_12 = x_25; goto block_15; } @@ -62205,13 +62205,13 @@ else { uint8_t x_26; x_26 = 0; -x_5 = x_16; -x_6 = x_17; -x_7 = x_18; -x_8 = x_22; -x_9 = x_19; -x_10 = lean_box(0); -x_11 = x_20; +x_5 = x_17; +x_6 = x_16; +x_7 = lean_box(0); +x_8 = x_18; +x_9 = x_22; +x_10 = x_20; +x_11 = x_21; x_12 = x_26; goto block_15; } @@ -62224,14 +62224,14 @@ lean_dec(x_31); if (lean_obj_tag(x_41) == 0) { lean_object* x_42; -lean_dec_ref(x_34); +lean_dec_ref(x_35); x_42 = l_Lean_Elab_elabAttrs___at___00Lean_Elab_elabDeclAttrs___at___00Lean_Elab_elabModifiers___at___00Lean_Elab_Command_elabMutualInductive_spec__0_spec__0_spec__1___closed__0; -x_16 = x_32; -x_17 = x_35; +x_16 = x_33; +x_17 = x_32; x_18 = x_36; x_19 = x_38; -x_20 = x_40; -x_21 = x_39; +x_20 = x_37; +x_21 = x_40; x_22 = x_42; x_23 = lean_box(0); goto block_27; @@ -62242,7 +62242,7 @@ lean_object* x_43; lean_object* x_44; x_43 = lean_ctor_get(x_41, 0); lean_inc(x_43); lean_dec_ref(x_41); -x_44 = l_Lean_Elab_elabDeclAttrs___at___00Lean_Elab_elabModifiers___at___00Lean_Elab_Command_elabMutualInductive_spec__0_spec__0(x_43, x_34, x_33); +x_44 = l_Lean_Elab_elabDeclAttrs___at___00Lean_Elab_elabModifiers___at___00Lean_Elab_Command_elabMutualInductive_spec__0_spec__0(x_43, x_35, x_34); lean_dec(x_43); if (lean_obj_tag(x_44) == 0) { @@ -62250,12 +62250,12 @@ lean_object* x_45; x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); lean_dec_ref(x_44); -x_16 = x_32; -x_17 = x_35; +x_16 = x_33; +x_17 = x_32; x_18 = x_36; x_19 = x_38; -x_20 = x_40; -x_21 = x_39; +x_20 = x_37; +x_21 = x_40; x_22 = x_45; x_23 = lean_box(0); goto block_27; @@ -62263,8 +62263,8 @@ goto block_27; else { uint8_t x_46; -lean_dec(x_39); -lean_dec(x_35); +lean_dec(x_38); +lean_dec(x_37); lean_dec(x_1); x_46 = !lean_is_exclusive(x_44); if (x_46 == 0) @@ -62294,13 +62294,13 @@ if (x_62 == 0) uint8_t x_63; x_63 = 1; x_32 = x_54; -x_33 = x_60; -x_34 = x_59; -x_35 = x_55; -x_36 = x_56; -x_37 = lean_box(0); -x_38 = x_58; -x_39 = x_57; +x_33 = x_58; +x_34 = x_60; +x_35 = x_59; +x_36 = x_55; +x_37 = x_57; +x_38 = x_56; +x_39 = lean_box(0); x_40 = x_63; goto block_49; } @@ -62309,13 +62309,13 @@ else uint8_t x_64; x_64 = 0; x_32 = x_54; -x_33 = x_60; -x_34 = x_59; -x_35 = x_55; -x_36 = x_56; -x_37 = lean_box(0); -x_38 = x_58; -x_39 = x_57; +x_33 = x_58; +x_34 = x_60; +x_35 = x_59; +x_36 = x_55; +x_37 = x_57; +x_38 = x_56; +x_39 = lean_box(0); x_40 = x_64; goto block_49; } @@ -62330,9 +62330,9 @@ if (lean_obj_tag(x_71) == 0) uint8_t x_72; x_72 = 0; x_54 = x_66; -x_55 = x_70; -x_56 = x_67; -x_57 = x_69; +x_55 = x_67; +x_56 = x_68; +x_57 = x_70; x_58 = x_72; x_59 = x_2; x_60 = x_3; @@ -62358,7 +62358,7 @@ if (x_77 == 0) { lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_dec(x_70); -lean_dec(x_69); +lean_dec(x_68); lean_dec(x_53); lean_dec(x_31); lean_dec(x_1); @@ -62387,9 +62387,9 @@ uint8_t x_83; lean_dec(x_73); x_83 = 2; x_54 = x_66; -x_55 = x_70; -x_56 = x_67; -x_57 = x_69; +x_55 = x_67; +x_56 = x_68; +x_57 = x_70; x_58 = x_83; x_59 = x_2; x_60 = x_3; @@ -62403,9 +62403,9 @@ uint8_t x_84; lean_dec(x_73); x_84 = 1; x_54 = x_66; -x_55 = x_70; -x_56 = x_67; -x_57 = x_69; +x_55 = x_67; +x_56 = x_68; +x_57 = x_70; x_58 = x_84; x_59 = x_2; x_60 = x_3; @@ -62436,8 +62436,8 @@ lean_dec(x_93); x_95 = lean_box(0); x_66 = x_88; x_67 = x_86; -x_68 = lean_box(0); -x_69 = x_87; +x_68 = x_87; +x_69 = lean_box(0); x_70 = x_95; goto block_85; } @@ -62459,8 +62459,8 @@ lean_ctor_set(x_101, 1, x_100); lean_ctor_set(x_94, 0, x_101); x_66 = x_88; x_67 = x_86; -x_68 = lean_box(0); -x_69 = x_87; +x_68 = x_87; +x_69 = lean_box(0); x_70 = x_94; goto block_85; } @@ -62481,8 +62481,8 @@ x_107 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_107, 0, x_106); x_66 = x_88; x_67 = x_86; -x_68 = lean_box(0); -x_69 = x_87; +x_68 = x_87; +x_69 = lean_box(0); x_70 = x_107; goto block_85; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c index 39579d6b8777..0cce937fddc9 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c @@ -603,7 +603,7 @@ goto block_19; if (x_10 == 0) { lean_object* x_11; lean_object* x_12; -lean_dec_ref(x_8); +lean_dec_ref(x_9); x_11 = lean_box(0); x_12 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_12, 0, x_11); @@ -611,7 +611,7 @@ return x_12; } else { -return x_8; +return x_9; } } block_19: @@ -622,16 +622,16 @@ if (x_17 == 0) { uint8_t x_18; x_18 = l_Lean_Exception_isRuntime(x_15); -x_8 = x_14; -x_9 = lean_box(0); +x_8 = lean_box(0); +x_9 = x_14; x_10 = x_18; goto block_13; } else { lean_dec_ref(x_15); -x_8 = x_14; -x_9 = lean_box(0); +x_8 = lean_box(0); +x_9 = x_14; x_10 = x_17; goto block_13; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c index 99735d09eaed..21814678af55 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c @@ -14179,7 +14179,7 @@ x_38 = l_WellFounded_opaqueFix_u2083___at___00Lean_Elab_Structural_getRecArgInfo x_39 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_39, 0, x_37); lean_ctor_set(x_39, 1, x_38); -x_40 = l_Lean_Exception_toMessageData(x_32); +x_40 = l_Lean_Exception_toMessageData(x_31); x_41 = l_Lean_indentD(x_40); x_42 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_42, 0, x_39); @@ -14198,7 +14198,7 @@ goto block_24; else { uint8_t x_46; -lean_dec_ref(x_32); +lean_dec_ref(x_31); lean_dec(x_27); lean_dec(x_16); lean_dec_ref(x_15); @@ -14245,7 +14245,7 @@ lean_dec_ref(x_4); lean_dec_ref(x_3); lean_dec(x_1); x_49 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_49, 0, x_32); +lean_ctor_set(x_49, 0, x_31); return x_49; } } @@ -14258,15 +14258,15 @@ if (x_53 == 0) uint8_t x_54; lean_inc_ref(x_51); x_54 = l_Lean_Exception_isRuntime(x_51); -x_31 = lean_box(0); -x_32 = x_51; +x_31 = x_51; +x_32 = lean_box(0); x_33 = x_54; goto block_50; } else { -x_31 = lean_box(0); -x_32 = x_51; +x_31 = x_51; +x_32 = lean_box(0); x_33 = x_53; goto block_50; } @@ -16902,18 +16902,18 @@ goto block_111; block_150: { lean_object* x_132; -lean_inc(x_128); -lean_inc_ref(x_124); -lean_inc(x_129); -lean_inc_ref(x_130); -x_132 = l_Lean_Elab_Structural_inductiveGroups(x_131, x_130, x_129, x_124, x_128); +lean_inc(x_124); +lean_inc_ref(x_127); +lean_inc(x_130); +lean_inc_ref(x_125); +x_132 = l_Lean_Elab_Structural_inductiveGroups(x_131, x_125, x_130, x_127, x_124); if (lean_obj_tag(x_132) == 0) { lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; x_133 = lean_ctor_get(x_132, 0); lean_inc(x_133); lean_dec_ref(x_132); -x_134 = l_Lean_isTracingEnabledFor___at___00Lean_Elab_Structural_tryAllArgs_spec__1___redArg(x_39, x_124); +x_134 = l_Lean_isTracingEnabledFor___at___00Lean_Elab_Structural_tryAllArgs_spec__1___redArg(x_39, x_127); x_135 = lean_ctor_get(x_134, 0); lean_inc(x_135); lean_dec_ref(x_134); @@ -16923,12 +16923,12 @@ if (x_136 == 0) { lean_dec(x_31); x_112 = x_133; -x_113 = x_125; -x_114 = x_126; -x_115 = x_130; -x_116 = x_129; -x_117 = x_124; -x_118 = x_128; +x_113 = x_128; +x_114 = x_129; +x_115 = x_125; +x_116 = x_130; +x_117 = x_127; +x_118 = x_124; x_119 = lean_box(0); goto block_123; } @@ -16949,17 +16949,17 @@ if (lean_is_scalar(x_31)) { } lean_ctor_set(x_142, 0, x_137); lean_ctor_set(x_142, 1, x_141); -x_143 = l_Lean_addTrace___at___00Lean_Elab_Structural_tryAllArgs_spec__3___redArg(x_39, x_142, x_130, x_129, x_124, x_128); +x_143 = l_Lean_addTrace___at___00Lean_Elab_Structural_tryAllArgs_spec__3___redArg(x_39, x_142, x_125, x_130, x_127, x_124); if (lean_obj_tag(x_143) == 0) { lean_dec_ref(x_143); x_112 = x_133; -x_113 = x_125; -x_114 = x_126; -x_115 = x_130; -x_116 = x_129; -x_117 = x_124; -x_118 = x_128; +x_113 = x_128; +x_114 = x_129; +x_115 = x_125; +x_116 = x_130; +x_117 = x_127; +x_118 = x_124; x_119 = lean_box(0); goto block_123; } @@ -16967,12 +16967,12 @@ else { uint8_t x_144; lean_dec(x_133); -lean_dec_ref(x_130); +lean_dec(x_130); lean_dec(x_129); -lean_dec(x_128); -lean_dec(x_126); +lean_dec_ref(x_128); +lean_dec_ref(x_127); lean_dec_ref(x_125); -lean_dec_ref(x_124); +lean_dec(x_124); lean_dec_ref(x_44); lean_dec(x_38); lean_dec(x_35); @@ -17001,12 +17001,12 @@ return x_146; else { uint8_t x_147; -lean_dec_ref(x_130); +lean_dec(x_130); lean_dec(x_129); -lean_dec(x_128); -lean_dec(x_126); +lean_dec_ref(x_128); +lean_dec_ref(x_127); lean_dec_ref(x_125); -lean_dec_ref(x_124); +lean_dec(x_124); lean_dec_ref(x_44); lean_dec(x_38); lean_dec(x_35); @@ -17040,13 +17040,13 @@ x_159 = lean_array_get_size(x_44); x_160 = lean_nat_dec_lt(x_14, x_159); if (x_160 == 0) { -x_124 = x_155; -x_125 = x_151; -x_126 = x_152; -x_127 = lean_box(0); -x_128 = x_156; -x_129 = x_154; -x_130 = x_153; +x_124 = x_156; +x_125 = x_153; +x_126 = lean_box(0); +x_127 = x_155; +x_128 = x_151; +x_129 = x_152; +x_130 = x_154; x_131 = x_158; goto block_150; } @@ -17056,13 +17056,13 @@ uint8_t x_161; x_161 = lean_nat_dec_le(x_159, x_159); if (x_161 == 0) { -x_124 = x_155; -x_125 = x_151; -x_126 = x_152; -x_127 = lean_box(0); -x_128 = x_156; -x_129 = x_154; -x_130 = x_153; +x_124 = x_156; +x_125 = x_153; +x_126 = lean_box(0); +x_127 = x_155; +x_128 = x_151; +x_129 = x_152; +x_130 = x_154; x_131 = x_158; goto block_150; } @@ -17071,13 +17071,13 @@ else size_t x_162; lean_object* x_163; x_162 = lean_usize_of_nat(x_159); x_163 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00Lean_Elab_Structural_tryAllArgs_spec__10(x_44, x_27, x_162, x_158); -x_124 = x_155; -x_125 = x_151; -x_126 = x_152; -x_127 = lean_box(0); -x_128 = x_156; -x_129 = x_154; -x_130 = x_153; +x_124 = x_156; +x_125 = x_153; +x_126 = lean_box(0); +x_127 = x_155; +x_128 = x_151; +x_129 = x_152; +x_130 = x_154; x_131 = x_163; goto block_150; } diff --git a/stage0/stdlib/Lean/Elab/Structure.c b/stage0/stdlib/Lean/Elab/Structure.c index c24c203c59cc..5089b9b271f9 100644 --- a/stage0/stdlib/Lean/Elab/Structure.c +++ b/stage0/stdlib/Lean/Elab/Structure.c @@ -42789,8 +42789,8 @@ lean_inc_ref(x_1); lean_inc(x_21); x_49 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___lam__0___boxed), 20, 11); lean_closure_set(x_49, 0, x_21); -lean_closure_set(x_49, 1, x_35); -lean_closure_set(x_49, 2, x_34); +lean_closure_set(x_49, 1, x_34); +lean_closure_set(x_49, 2, x_35); lean_closure_set(x_49, 3, x_5); lean_closure_set(x_49, 4, x_1); lean_closure_set(x_49, 5, x_2); @@ -42799,7 +42799,7 @@ lean_closure_set(x_49, 7, x_4); lean_closure_set(x_49, 8, x_22); lean_closure_set(x_49, 9, x_47); lean_closure_set(x_49, 10, x_48); -x_50 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParent___redArg(x_1, x_21, x_45, x_37, x_32, x_49, x_44, x_40, x_36, x_42, x_41, x_38, x_43); +x_50 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParent___redArg(x_1, x_21, x_40, x_45, x_32, x_49, x_37, x_44, x_38, x_39, x_36, x_42, x_41); return x_50; } block_95: @@ -42807,25 +42807,25 @@ return x_50; if (x_67 == 0) { lean_object* x_68; uint8_t x_69; -lean_dec(x_59); +lean_dec(x_65); lean_inc(x_21); -x_68 = lean_array_get_size(x_53); -x_69 = lean_nat_dec_lt(x_57, x_68); +x_68 = lean_array_get_size(x_52); +x_69 = lean_nat_dec_lt(x_60, x_68); if (x_69 == 0) { -lean_dec_ref(x_53); -x_34 = x_52; +lean_dec_ref(x_52); +x_34 = x_53; x_35 = x_54; -x_36 = x_60; -x_37 = x_61; -x_38 = x_55; -x_39 = lean_box(0); -x_40 = x_56; +x_36 = x_61; +x_37 = x_55; +x_38 = x_56; +x_39 = x_57; +x_40 = x_62; x_41 = x_63; x_42 = x_64; -x_43 = x_58; -x_44 = x_65; -x_45 = x_66; +x_43 = lean_box(0); +x_44 = x_66; +x_45 = x_59; x_46 = x_67; goto block_51; } @@ -42833,19 +42833,19 @@ else { if (x_69 == 0) { -lean_dec_ref(x_53); -x_34 = x_52; +lean_dec_ref(x_52); +x_34 = x_53; x_35 = x_54; -x_36 = x_60; -x_37 = x_61; -x_38 = x_55; -x_39 = lean_box(0); -x_40 = x_56; +x_36 = x_61; +x_37 = x_55; +x_38 = x_56; +x_39 = x_57; +x_40 = x_62; x_41 = x_63; x_42 = x_64; -x_43 = x_58; -x_44 = x_65; -x_45 = x_66; +x_43 = lean_box(0); +x_44 = x_66; +x_45 = x_59; x_46 = x_67; goto block_51; } @@ -42854,34 +42854,34 @@ else size_t x_70; size_t x_71; uint8_t x_72; x_70 = 0; x_71 = lean_usize_of_nat(x_68); -x_72 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__0(x_61, x_53, x_70, x_71); -lean_dec_ref(x_53); +x_72 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__0(x_59, x_52, x_70, x_71); +lean_dec_ref(x_52); if (x_72 == 0) { -x_34 = x_52; +x_34 = x_53; x_35 = x_54; -x_36 = x_60; -x_37 = x_61; -x_38 = x_55; -x_39 = lean_box(0); -x_40 = x_56; +x_36 = x_61; +x_37 = x_55; +x_38 = x_56; +x_39 = x_57; +x_40 = x_62; x_41 = x_63; x_42 = x_64; -x_43 = x_58; -x_44 = x_65; -x_45 = x_66; +x_43 = lean_box(0); +x_44 = x_66; +x_45 = x_59; x_46 = x_72; goto block_51; } else { lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_66); -lean_dec_ref(x_65); -lean_dec(x_60); -lean_dec_ref(x_56); +lean_dec_ref(x_66); +lean_dec(x_62); +lean_dec(x_56); +lean_dec_ref(x_55); lean_dec(x_54); -lean_dec(x_52); +lean_dec(x_53); lean_dec(x_32); lean_dec(x_21); lean_dec(x_5); @@ -42890,7 +42890,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_73 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withStruct___redArg___lam__1___closed__1; -x_74 = l_Lean_MessageData_ofName(x_61); +x_74 = l_Lean_MessageData_ofName(x_59); x_75 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_75, 0, x_73); lean_ctor_set(x_75, 1, x_74); @@ -42902,11 +42902,11 @@ x_78 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withStruct x_79 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_79, 0, x_77); lean_ctor_set(x_79, 1, x_78); -x_80 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_79, x_64, x_63, x_55, x_58); -lean_dec(x_58); -lean_dec_ref(x_55); +x_80 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_79, x_57, x_61, x_64, x_63); lean_dec(x_63); lean_dec_ref(x_64); +lean_dec(x_61); +lean_dec_ref(x_57); return x_80; } } @@ -42915,14 +42915,14 @@ return x_80; 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_dec(x_66); -lean_dec(x_61); +lean_dec(x_62); +lean_dec(x_59); lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); +lean_dec(x_53); +lean_dec_ref(x_52); lean_dec(x_32); x_81 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___closed__1; -x_82 = l_Lean_MessageData_ofConstName(x_59, x_29); +x_82 = l_Lean_MessageData_ofConstName(x_65, x_29); x_83 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_83, 0, x_81); lean_ctor_set(x_83, 1, x_82); @@ -42930,8 +42930,8 @@ x_84 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParent x_85 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); -lean_inc_ref(x_55); -x_86 = l_Lean_logWarning___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__1(x_85, x_65, x_56, x_60, x_64, x_63, x_55, x_58); +lean_inc_ref(x_64); +x_86 = l_Lean_logWarning___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__1(x_85, x_55, x_66, x_56, x_57, x_61, x_64, x_63); if (lean_obj_tag(x_86) == 0) { lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; @@ -42946,23 +42946,23 @@ x_90 = lean_nat_add(x_5, x_89); lean_dec(x_5); x_5 = x_90; x_6 = x_88; -x_7 = x_56; -x_8 = x_60; -x_9 = x_64; -x_10 = x_63; -x_11 = x_55; -x_12 = x_58; +x_7 = x_66; +x_8 = x_56; +x_9 = x_57; +x_10 = x_61; +x_11 = x_64; +x_12 = x_63; goto _start; } else { uint8_t x_92; +lean_dec_ref(x_66); lean_dec_ref(x_64); lean_dec(x_63); -lean_dec(x_60); -lean_dec(x_58); -lean_dec_ref(x_56); -lean_dec_ref(x_55); +lean_dec(x_61); +lean_dec_ref(x_57); +lean_dec(x_56); lean_dec(x_5); lean_dec_ref(x_4); lean_dec_ref(x_3); @@ -43003,23 +43003,23 @@ x_112 = lean_array_get_size(x_110); x_113 = lean_nat_dec_lt(x_111, x_112); if (x_113 == 0) { -lean_inc(x_104); lean_inc(x_109); -x_52 = x_109; -x_53 = x_110; -x_54 = x_104; -x_55 = x_99; -x_56 = x_100; -x_57 = x_111; -x_58 = x_103; -x_59 = x_104; -x_60 = x_98; -x_61 = x_109; -x_62 = lean_box(0); +lean_inc(x_104); +x_52 = x_110; +x_53 = x_104; +x_54 = x_109; +x_55 = x_105; +x_56 = x_99; +x_57 = x_100; +x_58 = lean_box(0); +x_59 = x_109; +x_60 = x_111; +x_61 = x_98; +x_62 = x_108; x_63 = x_101; x_64 = x_102; -x_65 = x_105; -x_66 = x_108; +x_65 = x_104; +x_66 = x_103; x_67 = x_97; goto block_95; } @@ -43027,23 +43027,23 @@ else { if (x_113 == 0) { -lean_inc(x_104); lean_inc(x_109); -x_52 = x_109; -x_53 = x_110; -x_54 = x_104; -x_55 = x_99; -x_56 = x_100; -x_57 = x_111; -x_58 = x_103; -x_59 = x_104; -x_60 = x_98; -x_61 = x_109; -x_62 = lean_box(0); +lean_inc(x_104); +x_52 = x_110; +x_53 = x_104; +x_54 = x_109; +x_55 = x_105; +x_56 = x_99; +x_57 = x_100; +x_58 = lean_box(0); +x_59 = x_109; +x_60 = x_111; +x_61 = x_98; +x_62 = x_108; x_63 = x_101; x_64 = x_102; -x_65 = x_105; -x_66 = x_108; +x_65 = x_104; +x_66 = x_103; x_67 = x_97; goto block_95; } @@ -43053,23 +43053,23 @@ size_t x_114; size_t x_115; uint8_t x_116; x_114 = 0; x_115 = lean_usize_of_nat(x_112); x_116 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__1(x_104, x_110, x_114, x_115); -lean_inc(x_104); lean_inc(x_109); -x_52 = x_109; -x_53 = x_110; -x_54 = x_104; -x_55 = x_99; -x_56 = x_100; -x_57 = x_111; -x_58 = x_103; -x_59 = x_104; -x_60 = x_98; -x_61 = x_109; -x_62 = lean_box(0); +lean_inc(x_104); +x_52 = x_110; +x_53 = x_104; +x_54 = x_109; +x_55 = x_105; +x_56 = x_99; +x_57 = x_100; +x_58 = lean_box(0); +x_59 = x_109; +x_60 = x_111; +x_61 = x_98; +x_62 = x_108; x_63 = x_101; x_64 = x_102; -x_65 = x_105; -x_66 = x_108; +x_65 = x_104; +x_66 = x_103; x_67 = x_116; goto block_95; } @@ -43077,21 +43077,21 @@ goto block_95; } block_135: { -lean_dec_ref(x_121); -lean_dec(x_118); +lean_dec_ref(x_125); +lean_dec(x_119); if (x_126 == 0) { lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_dec(x_33); -x_127 = l_Lean_Exception_toMessageData(x_125); +x_127 = l_Lean_Exception_toMessageData(x_123); x_128 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___closed__7; x_129 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_129, 0, x_127); lean_ctor_set(x_129, 1, x_128); -x_130 = l_Lean_throwErrorAt___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_instantiateStructDefaultValueFn_x3f___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__0_spec__0_spec__1_spec__4_spec__9_spec__12___redArg(x_23, x_129, x_123, x_122, x_120, x_124); -lean_dec(x_124); +x_130 = l_Lean_throwErrorAt___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_instantiateStructDefaultValueFn_x3f___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__0_spec__0_spec__1_spec__4_spec__9_spec__12___redArg(x_23, x_129, x_121, x_118, x_124, x_122); lean_dec(x_122); -lean_dec_ref(x_123); +lean_dec(x_118); +lean_dec_ref(x_121); lean_dec(x_23); x_131 = !lean_is_exclusive(x_130); if (x_131 == 0) @@ -43112,10 +43112,10 @@ return x_133; else { lean_object* x_134; -lean_dec(x_124); -lean_dec_ref(x_123); +lean_dec_ref(x_124); lean_dec(x_122); -lean_dec_ref(x_120); +lean_dec_ref(x_121); +lean_dec(x_118); lean_dec(x_23); if (lean_is_scalar(x_33)) { x_134 = lean_alloc_ctor(1, 1, 0); @@ -43123,7 +43123,7 @@ if (lean_is_scalar(x_33)) { x_134 = x_33; lean_ctor_set_tag(x_134, 1); } -lean_ctor_set(x_134, 0, x_125); +lean_ctor_set(x_134, 0, x_123); return x_134; } } @@ -43138,12 +43138,12 @@ lean_dec(x_33); x_145 = lean_ctor_get(x_144, 0); lean_inc(x_145); lean_dec_ref(x_144); -x_98 = x_138; -x_99 = x_141; -x_100 = x_137; -x_101 = x_140; -x_102 = x_139; -x_103 = x_142; +x_98 = x_140; +x_99 = x_138; +x_100 = x_139; +x_101 = x_142; +x_102 = x_141; +x_103 = x_137; x_104 = x_145; x_105 = x_136; x_106 = lean_box(0); @@ -43169,27 +43169,27 @@ if (x_147 == 0) uint8_t x_148; lean_inc(x_146); x_148 = l_Lean_Exception_isRuntime(x_146); -x_118 = x_138; -x_119 = lean_box(0); -x_120 = x_141; -x_121 = x_137; -x_122 = x_140; -x_123 = x_139; -x_124 = x_142; -x_125 = x_146; +x_118 = x_140; +x_119 = x_138; +x_120 = lean_box(0); +x_121 = x_139; +x_122 = x_142; +x_123 = x_146; +x_124 = x_141; +x_125 = x_137; x_126 = x_148; goto block_135; } else { -x_118 = x_138; -x_119 = lean_box(0); -x_120 = x_141; -x_121 = x_137; -x_122 = x_140; -x_123 = x_139; -x_124 = x_142; -x_125 = x_146; +x_118 = x_140; +x_119 = x_138; +x_120 = lean_box(0); +x_121 = x_139; +x_122 = x_142; +x_123 = x_146; +x_124 = x_141; +x_125 = x_137; x_126 = x_147; goto block_135; } @@ -43544,8 +43544,8 @@ lean_inc_ref(x_1); lean_inc(x_183); x_227 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___lam__0___boxed), 20, 11); lean_closure_set(x_227, 0, x_183); -lean_closure_set(x_227, 1, x_213); -lean_closure_set(x_227, 2, x_212); +lean_closure_set(x_227, 1, x_212); +lean_closure_set(x_227, 2, x_213); lean_closure_set(x_227, 3, x_5); lean_closure_set(x_227, 4, x_1); lean_closure_set(x_227, 5, x_2); @@ -43554,7 +43554,7 @@ lean_closure_set(x_227, 7, x_4); lean_closure_set(x_227, 8, x_184); lean_closure_set(x_227, 9, x_225); lean_closure_set(x_227, 10, x_226); -x_228 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParent___redArg(x_1, x_183, x_223, x_215, x_210, x_227, x_222, x_218, x_214, x_220, x_219, x_216, x_221); +x_228 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParent___redArg(x_1, x_183, x_218, x_223, x_210, x_227, x_215, x_222, x_216, x_217, x_214, x_220, x_219); return x_228; } block_273: @@ -43562,25 +43562,25 @@ return x_228; if (x_245 == 0) { lean_object* x_246; uint8_t x_247; -lean_dec(x_237); +lean_dec(x_243); lean_inc(x_183); -x_246 = lean_array_get_size(x_231); -x_247 = lean_nat_dec_lt(x_235, x_246); +x_246 = lean_array_get_size(x_230); +x_247 = lean_nat_dec_lt(x_238, x_246); if (x_247 == 0) { -lean_dec_ref(x_231); -x_212 = x_230; +lean_dec_ref(x_230); +x_212 = x_231; x_213 = x_232; -x_214 = x_238; -x_215 = x_239; -x_216 = x_233; -x_217 = lean_box(0); -x_218 = x_234; +x_214 = x_239; +x_215 = x_233; +x_216 = x_234; +x_217 = x_235; +x_218 = x_240; x_219 = x_241; x_220 = x_242; -x_221 = x_236; -x_222 = x_243; -x_223 = x_244; +x_221 = lean_box(0); +x_222 = x_244; +x_223 = x_237; x_224 = x_245; goto block_229; } @@ -43588,19 +43588,19 @@ else { if (x_247 == 0) { -lean_dec_ref(x_231); -x_212 = x_230; +lean_dec_ref(x_230); +x_212 = x_231; x_213 = x_232; -x_214 = x_238; -x_215 = x_239; -x_216 = x_233; -x_217 = lean_box(0); -x_218 = x_234; +x_214 = x_239; +x_215 = x_233; +x_216 = x_234; +x_217 = x_235; +x_218 = x_240; x_219 = x_241; x_220 = x_242; -x_221 = x_236; -x_222 = x_243; -x_223 = x_244; +x_221 = lean_box(0); +x_222 = x_244; +x_223 = x_237; x_224 = x_245; goto block_229; } @@ -43609,34 +43609,34 @@ else size_t x_248; size_t x_249; uint8_t x_250; x_248 = 0; x_249 = lean_usize_of_nat(x_246); -x_250 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__0(x_239, x_231, x_248, x_249); -lean_dec_ref(x_231); +x_250 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__0(x_237, x_230, x_248, x_249); +lean_dec_ref(x_230); if (x_250 == 0) { -x_212 = x_230; +x_212 = x_231; x_213 = x_232; -x_214 = x_238; -x_215 = x_239; -x_216 = x_233; -x_217 = lean_box(0); -x_218 = x_234; +x_214 = x_239; +x_215 = x_233; +x_216 = x_234; +x_217 = x_235; +x_218 = x_240; x_219 = x_241; x_220 = x_242; -x_221 = x_236; -x_222 = x_243; -x_223 = x_244; +x_221 = lean_box(0); +x_222 = x_244; +x_223 = x_237; x_224 = x_250; goto block_229; } else { 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_dec(x_244); -lean_dec_ref(x_243); -lean_dec(x_238); -lean_dec_ref(x_234); +lean_dec_ref(x_244); +lean_dec(x_240); +lean_dec(x_234); +lean_dec_ref(x_233); lean_dec(x_232); -lean_dec(x_230); +lean_dec(x_231); lean_dec(x_210); lean_dec(x_183); lean_dec(x_5); @@ -43645,7 +43645,7 @@ lean_dec_ref(x_3); lean_dec_ref(x_2); lean_dec_ref(x_1); x_251 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withStruct___redArg___lam__1___closed__1; -x_252 = l_Lean_MessageData_ofName(x_239); +x_252 = l_Lean_MessageData_ofName(x_237); x_253 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_253, 0, x_251); lean_ctor_set(x_253, 1, x_252); @@ -43657,11 +43657,11 @@ x_256 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withStruc x_257 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_257, 0, x_255); lean_ctor_set(x_257, 1, x_256); -x_258 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_257, x_242, x_241, x_233, x_236); -lean_dec(x_236); -lean_dec_ref(x_233); +x_258 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_257, x_235, x_239, x_242, x_241); lean_dec(x_241); lean_dec_ref(x_242); +lean_dec(x_239); +lean_dec_ref(x_235); return x_258; } } @@ -43670,14 +43670,14 @@ return x_258; else { 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_dec(x_244); -lean_dec(x_239); +lean_dec(x_240); +lean_dec(x_237); lean_dec(x_232); -lean_dec_ref(x_231); -lean_dec(x_230); +lean_dec(x_231); +lean_dec_ref(x_230); lean_dec(x_210); x_259 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___closed__1; -x_260 = l_Lean_MessageData_ofConstName(x_237, x_207); +x_260 = l_Lean_MessageData_ofConstName(x_243, x_207); x_261 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_261, 0, x_259); lean_ctor_set(x_261, 1, x_260); @@ -43685,8 +43685,8 @@ x_262 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParen x_263 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_263, 0, x_261); lean_ctor_set(x_263, 1, x_262); -lean_inc_ref(x_233); -x_264 = l_Lean_logWarning___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__1(x_263, x_243, x_234, x_238, x_242, x_241, x_233, x_236); +lean_inc_ref(x_242); +x_264 = l_Lean_logWarning___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__1(x_263, x_233, x_244, x_234, x_235, x_239, x_242, x_241); if (lean_obj_tag(x_264) == 0) { lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; @@ -43701,23 +43701,23 @@ x_268 = lean_nat_add(x_5, x_267); lean_dec(x_5); x_5 = x_268; x_6 = x_266; -x_7 = x_234; -x_8 = x_238; -x_9 = x_242; -x_10 = x_241; -x_11 = x_233; -x_12 = x_236; +x_7 = x_244; +x_8 = x_234; +x_9 = x_235; +x_10 = x_239; +x_11 = x_242; +x_12 = x_241; goto _start; } else { lean_object* x_270; lean_object* x_271; lean_object* x_272; +lean_dec_ref(x_244); lean_dec_ref(x_242); lean_dec(x_241); -lean_dec(x_238); -lean_dec(x_236); -lean_dec_ref(x_234); -lean_dec_ref(x_233); +lean_dec(x_239); +lean_dec_ref(x_235); +lean_dec(x_234); lean_dec(x_5); lean_dec_ref(x_4); lean_dec_ref(x_3); @@ -43759,23 +43759,23 @@ x_290 = lean_array_get_size(x_288); x_291 = lean_nat_dec_lt(x_289, x_290); if (x_291 == 0) { -lean_inc(x_282); lean_inc(x_287); -x_230 = x_287; -x_231 = x_288; -x_232 = x_282; -x_233 = x_277; -x_234 = x_278; -x_235 = x_289; -x_236 = x_281; -x_237 = x_282; -x_238 = x_276; -x_239 = x_287; -x_240 = lean_box(0); +lean_inc(x_282); +x_230 = x_288; +x_231 = x_282; +x_232 = x_287; +x_233 = x_283; +x_234 = x_277; +x_235 = x_278; +x_236 = lean_box(0); +x_237 = x_287; +x_238 = x_289; +x_239 = x_276; +x_240 = x_286; x_241 = x_279; x_242 = x_280; -x_243 = x_283; -x_244 = x_286; +x_243 = x_282; +x_244 = x_281; x_245 = x_275; goto block_273; } @@ -43783,23 +43783,23 @@ else { if (x_291 == 0) { -lean_inc(x_282); lean_inc(x_287); -x_230 = x_287; -x_231 = x_288; -x_232 = x_282; -x_233 = x_277; -x_234 = x_278; -x_235 = x_289; -x_236 = x_281; -x_237 = x_282; -x_238 = x_276; -x_239 = x_287; -x_240 = lean_box(0); +lean_inc(x_282); +x_230 = x_288; +x_231 = x_282; +x_232 = x_287; +x_233 = x_283; +x_234 = x_277; +x_235 = x_278; +x_236 = lean_box(0); +x_237 = x_287; +x_238 = x_289; +x_239 = x_276; +x_240 = x_286; x_241 = x_279; x_242 = x_280; -x_243 = x_283; -x_244 = x_286; +x_243 = x_282; +x_244 = x_281; x_245 = x_275; goto block_273; } @@ -43809,23 +43809,23 @@ size_t x_292; size_t x_293; uint8_t x_294; x_292 = 0; x_293 = lean_usize_of_nat(x_290); x_294 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go_spec__1(x_282, x_288, x_292, x_293); -lean_inc(x_282); lean_inc(x_287); -x_230 = x_287; -x_231 = x_288; -x_232 = x_282; -x_233 = x_277; -x_234 = x_278; -x_235 = x_289; -x_236 = x_281; -x_237 = x_282; -x_238 = x_276; -x_239 = x_287; -x_240 = lean_box(0); +lean_inc(x_282); +x_230 = x_288; +x_231 = x_282; +x_232 = x_287; +x_233 = x_283; +x_234 = x_277; +x_235 = x_278; +x_236 = lean_box(0); +x_237 = x_287; +x_238 = x_289; +x_239 = x_276; +x_240 = x_286; x_241 = x_279; x_242 = x_280; -x_243 = x_283; -x_244 = x_286; +x_243 = x_282; +x_244 = x_281; x_245 = x_294; goto block_273; } @@ -43833,21 +43833,21 @@ goto block_273; } block_313: { -lean_dec_ref(x_299); -lean_dec(x_296); +lean_dec_ref(x_303); +lean_dec(x_297); if (x_304 == 0) { 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_dec(x_211); -x_305 = l_Lean_Exception_toMessageData(x_303); +x_305 = l_Lean_Exception_toMessageData(x_301); x_306 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withParents_go___redArg___closed__7; x_307 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_307, 0, x_305); lean_ctor_set(x_307, 1, x_306); -x_308 = l_Lean_throwErrorAt___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_instantiateStructDefaultValueFn_x3f___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__0_spec__0_spec__1_spec__4_spec__9_spec__12___redArg(x_185, x_307, x_301, x_300, x_298, x_302); -lean_dec(x_302); +x_308 = l_Lean_throwErrorAt___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_instantiateStructDefaultValueFn_x3f___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_getFieldDefaultValue_x3f_spec__0_spec__0_spec__1_spec__4_spec__9_spec__12___redArg(x_185, x_307, x_299, x_296, x_302, x_300); lean_dec(x_300); -lean_dec_ref(x_301); +lean_dec(x_296); +lean_dec_ref(x_299); lean_dec(x_185); x_309 = lean_ctor_get(x_308, 0); lean_inc(x_309); @@ -43869,10 +43869,10 @@ return x_311; else { lean_object* x_312; -lean_dec(x_302); -lean_dec_ref(x_301); +lean_dec_ref(x_302); lean_dec(x_300); -lean_dec_ref(x_298); +lean_dec_ref(x_299); +lean_dec(x_296); lean_dec(x_185); if (lean_is_scalar(x_211)) { x_312 = lean_alloc_ctor(1, 1, 0); @@ -43880,7 +43880,7 @@ if (lean_is_scalar(x_211)) { x_312 = x_211; lean_ctor_set_tag(x_312, 1); } -lean_ctor_set(x_312, 0, x_303); +lean_ctor_set(x_312, 0, x_301); return x_312; } } @@ -43895,12 +43895,12 @@ lean_dec(x_211); x_323 = lean_ctor_get(x_322, 0); lean_inc(x_323); lean_dec_ref(x_322); -x_276 = x_316; -x_277 = x_319; -x_278 = x_315; -x_279 = x_318; -x_280 = x_317; -x_281 = x_320; +x_276 = x_318; +x_277 = x_316; +x_278 = x_317; +x_279 = x_320; +x_280 = x_319; +x_281 = x_315; x_282 = x_323; x_283 = x_314; x_284 = lean_box(0); @@ -43926,27 +43926,27 @@ if (x_325 == 0) uint8_t x_326; lean_inc(x_324); x_326 = l_Lean_Exception_isRuntime(x_324); -x_296 = x_316; -x_297 = lean_box(0); -x_298 = x_319; -x_299 = x_315; -x_300 = x_318; -x_301 = x_317; -x_302 = x_320; -x_303 = x_324; +x_296 = x_318; +x_297 = x_316; +x_298 = lean_box(0); +x_299 = x_317; +x_300 = x_320; +x_301 = x_324; +x_302 = x_319; +x_303 = x_315; x_304 = x_326; goto block_313; } else { -x_296 = x_316; -x_297 = lean_box(0); -x_298 = x_319; -x_299 = x_315; -x_300 = x_318; -x_301 = x_317; -x_302 = x_320; -x_303 = x_324; +x_296 = x_318; +x_297 = x_316; +x_298 = lean_box(0); +x_299 = x_317; +x_300 = x_320; +x_301 = x_324; +x_302 = x_319; +x_303 = x_315; x_304 = x_325; goto block_313; } @@ -55718,7 +55718,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withFields_go___redArg___lam__3(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, uint8_t 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) { _start: { -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_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_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_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; uint8_t x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_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_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_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_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_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; uint8_t 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_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; uint8_t 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_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; uint8_t x_609; +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_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_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_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_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_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_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_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_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; uint8_t 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_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; uint8_t 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_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; uint8_t x_609; x_609 = !lean_is_exclusive(x_22); if (x_609 == 0) { @@ -56327,23 +56327,23 @@ goto block_59; { lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; x_103 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_103, 0, x_89); +lean_ctor_set(x_103, 0, x_94); x_104 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_104, 0, x_103); x_105 = lean_alloc_ctor(0, 12, 1); lean_ctor_set(x_105, 0, x_8); -lean_ctor_set(x_105, 1, x_83); -lean_ctor_set(x_105, 2, x_88); -lean_ctor_set(x_105, 3, x_92); -lean_ctor_set(x_105, 4, x_91); -lean_ctor_set(x_105, 5, x_87); -lean_ctor_set(x_105, 6, x_90); +lean_ctor_set(x_105, 1, x_92); +lean_ctor_set(x_105, 2, x_89); +lean_ctor_set(x_105, 3, x_87); +lean_ctor_set(x_105, 4, x_85); +lean_ctor_set(x_105, 5, x_88); +lean_ctor_set(x_105, 6, x_91); lean_ctor_set(x_105, 7, x_93); lean_ctor_set(x_105, 8, x_104); -lean_ctor_set(x_105, 9, x_85); +lean_ctor_set(x_105, 9, x_83); lean_ctor_set(x_105, 10, x_84); -lean_ctor_set(x_105, 11, x_86); -lean_ctor_set_uint8(x_105, sizeof(void*)*12, x_94); +lean_ctor_set(x_105, 11, x_90); +lean_ctor_set_uint8(x_105, sizeof(void*)*12, x_86); x_106 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_105, x_95, x_98, x_99, x_100, x_101); if (lean_obj_tag(x_106) == 0) { @@ -56493,18 +56493,18 @@ x_155 = l_Lean_Elab_Term_addTermInfo_x27(x_10, x_151, x_140, x_140, x_153, x_154 if (lean_obj_tag(x_155) == 0) { lean_dec_ref(x_155); -x_83 = x_126; +x_83 = x_134; x_84 = x_135; -x_85 = x_134; -x_86 = x_136; -x_87 = x_131; -x_88 = x_127; -x_89 = x_142; -x_90 = x_132; -x_91 = x_130; -x_92 = x_128; +x_85 = x_130; +x_86 = x_129; +x_87 = x_128; +x_88 = x_131; +x_89 = x_127; +x_90 = x_136; +x_91 = x_132; +x_92 = x_126; x_93 = x_133; -x_94 = x_129; +x_94 = x_142; x_95 = x_152; x_96 = x_119; x_97 = x_120; @@ -56608,18 +56608,18 @@ lean_dec(x_10); x_162 = lean_ctor_get(x_146, 1); lean_inc(x_162); lean_dec(x_146); -x_83 = x_126; +x_83 = x_134; x_84 = x_135; -x_85 = x_134; -x_86 = x_136; -x_87 = x_131; -x_88 = x_127; -x_89 = x_142; -x_90 = x_132; -x_91 = x_130; -x_92 = x_128; +x_85 = x_130; +x_86 = x_129; +x_87 = x_128; +x_88 = x_131; +x_89 = x_127; +x_90 = x_136; +x_91 = x_132; +x_92 = x_126; x_93 = x_133; -x_94 = x_129; +x_94 = x_142; x_95 = x_162; x_96 = x_119; x_97 = x_120; @@ -56888,7 +56888,7 @@ x_222 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withField x_223 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_223, 0, x_222); lean_ctor_set(x_223, 1, x_221); -x_224 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_223, x_213, x_212, x_208, x_210); +x_224 = l_Lean_throwError___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addFieldInfo_spec__0___redArg(x_223, x_212, x_214, x_211, x_213); if (lean_obj_tag(x_224) == 0) { lean_object* x_225; lean_object* x_226; @@ -56898,31 +56898,31 @@ lean_dec_ref(x_224); x_226 = lean_ctor_get(x_225, 1); lean_inc(x_226); lean_dec(x_225); -x_176 = x_209; -x_177 = x_211; -x_178 = x_207; +x_176 = x_208; +x_177 = x_207; +x_178 = x_215; x_179 = x_226; -x_180 = x_215; -x_181 = x_214; -x_182 = x_213; -x_183 = x_212; -x_184 = x_208; -x_185 = x_210; +x_180 = x_216; +x_181 = x_210; +x_182 = x_212; +x_183 = x_214; +x_184 = x_211; +x_185 = x_213; x_186 = lean_box(0); goto block_206; } else { uint8_t x_227; -lean_dec_ref(x_215); +lean_dec_ref(x_216); +lean_dec(x_215); lean_dec(x_214); -lean_dec_ref(x_213); -lean_dec(x_212); +lean_dec(x_213); +lean_dec_ref(x_212); lean_dec_ref(x_211); lean_dec(x_210); -lean_dec_ref(x_209); lean_dec_ref(x_208); -lean_dec(x_207); +lean_dec_ref(x_207); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); @@ -56993,16 +56993,16 @@ x_254 = lean_nat_dec_lt(x_250, x_253); if (x_254 == 0) { lean_dec_ref(x_249); -x_207 = x_231; -x_208 = x_238; -x_209 = x_232; -x_210 = x_239; -x_211 = x_247; -x_212 = x_237; -x_213 = x_236; -x_214 = x_235; -x_215 = x_234; -x_216 = lean_box(0); +x_207 = x_247; +x_208 = x_231; +x_209 = lean_box(0); +x_210 = x_235; +x_211 = x_238; +x_212 = x_236; +x_213 = x_239; +x_214 = x_237; +x_215 = x_232; +x_216 = x_234; x_217 = x_252; goto block_230; } @@ -57013,16 +57013,16 @@ x_255 = lean_usize_of_nat(x_253); x_256 = 0; x_257 = l___private_Init_Data_Array_Basic_0__Array_foldrMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withFields_go_spec__3(x_249, x_255, x_256, x_252); lean_dec_ref(x_249); -x_207 = x_231; -x_208 = x_238; -x_209 = x_232; -x_210 = x_239; -x_211 = x_247; -x_212 = x_237; -x_213 = x_236; -x_214 = x_235; -x_215 = x_234; -x_216 = lean_box(0); +x_207 = x_247; +x_208 = x_231; +x_209 = lean_box(0); +x_210 = x_235; +x_211 = x_238; +x_212 = x_236; +x_213 = x_239; +x_214 = x_237; +x_215 = x_232; +x_216 = x_234; x_217 = x_257; goto block_230; } @@ -57030,9 +57030,9 @@ goto block_230; else { lean_dec_ref(x_249); -x_176 = x_232; +x_176 = x_231; x_177 = x_247; -x_178 = x_231; +x_178 = x_232; x_179 = x_246; x_180 = x_234; x_181 = x_235; @@ -57053,8 +57053,8 @@ lean_dec(x_237); lean_dec_ref(x_236); lean_dec(x_235); lean_dec_ref(x_234); -lean_dec_ref(x_232); -lean_dec(x_231); +lean_dec(x_232); +lean_dec_ref(x_231); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); @@ -57090,7 +57090,7 @@ lean_inc(x_280); lean_inc_ref(x_279); lean_inc(x_278); lean_inc_ref(x_277); -x_284 = l_Lean_Elab_Term_declareTacticSyntax(x_273, x_283, x_275, x_276, x_277, x_278, x_279, x_280); +x_284 = l_Lean_Elab_Term_declareTacticSyntax(x_268, x_283, x_275, x_276, x_277, x_278, x_279, x_280); if (lean_obj_tag(x_284) == 0) { lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; @@ -57101,21 +57101,21 @@ x_287 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_287, 0, x_286); x_288 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_288, 0, x_287); -lean_inc(x_264); +lean_inc(x_269); x_289 = lean_alloc_ctor(0, 12, 1); lean_ctor_set(x_289, 0, x_8); -lean_ctor_set(x_289, 1, x_268); -lean_ctor_set(x_289, 2, x_262); -lean_ctor_set(x_289, 3, x_265); -lean_ctor_set(x_289, 4, x_267); -lean_ctor_set(x_289, 5, x_266); -lean_ctor_set(x_289, 6, x_271); -lean_ctor_set(x_289, 7, x_270); +lean_ctor_set(x_289, 1, x_264); +lean_ctor_set(x_289, 2, x_270); +lean_ctor_set(x_289, 3, x_266); +lean_ctor_set(x_289, 4, x_273); +lean_ctor_set(x_289, 5, x_262); +lean_ctor_set(x_289, 6, x_267); +lean_ctor_set(x_289, 7, x_265); lean_ctor_set(x_289, 8, x_288); -lean_ctor_set(x_289, 9, x_264); -lean_ctor_set(x_289, 10, x_269); +lean_ctor_set(x_289, 9, x_269); +lean_ctor_set(x_289, 10, x_272); lean_ctor_set(x_289, 11, x_263); -lean_ctor_set_uint8(x_289, sizeof(void*)*12, x_272); +lean_ctor_set_uint8(x_289, sizeof(void*)*12, x_271); x_290 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_289, x_274, x_277, x_278, x_279, x_280); if (lean_obj_tag(x_290) == 0) { @@ -57136,15 +57136,15 @@ lean_object* x_295; x_295 = lean_ctor_get(x_294, 0); lean_inc(x_295); lean_dec_ref(x_294); -if (lean_obj_tag(x_264) == 1) +if (lean_obj_tag(x_269) == 1) { lean_object* x_296; lean_object* x_297; lean_object* x_298; x_296 = lean_ctor_get(x_295, 1); lean_inc(x_296); lean_dec(x_295); -x_297 = lean_ctor_get(x_264, 0); +x_297 = lean_ctor_get(x_269, 0); lean_inc(x_297); -lean_dec_ref(x_264); +lean_dec_ref(x_269); lean_inc_ref(x_279); x_298 = l_Lean_mkConstWithLevelParams___at___00Lean_Elab_checkNotAlreadyDeclared___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_withStruct_spec__2_spec__2(x_297, x_296, x_275, x_276, x_277, x_278, x_279, x_280); if (lean_obj_tag(x_298) == 0) @@ -57246,7 +57246,7 @@ return x_311; else { lean_object* x_312; -lean_dec(x_264); +lean_dec(x_269); lean_dec(x_10); x_312 = lean_ctor_get(x_295, 1); lean_inc(x_312); @@ -57271,7 +57271,7 @@ lean_dec(x_278); lean_dec_ref(x_277); lean_dec(x_276); lean_dec_ref(x_275); -lean_dec(x_264); +lean_dec(x_269); lean_dec(x_10); lean_dec_ref(x_5); lean_dec_ref(x_4); @@ -57303,7 +57303,7 @@ lean_dec(x_278); lean_dec_ref(x_277); lean_dec(x_276); lean_dec_ref(x_275); -lean_dec(x_264); +lean_dec(x_269); lean_dec(x_10); lean_dec_ref(x_5); lean_dec_ref(x_4); @@ -57337,10 +57337,10 @@ lean_dec_ref(x_277); lean_dec(x_276); lean_dec_ref(x_275); lean_dec_ref(x_274); -lean_dec_ref(x_271); +lean_dec_ref(x_273); +lean_dec_ref(x_272); lean_dec(x_270); -lean_dec_ref(x_269); -lean_dec(x_268); +lean_dec(x_269); lean_dec_ref(x_267); lean_dec(x_266); lean_dec(x_265); @@ -57381,17 +57381,17 @@ x_346 = lean_nat_dec_lt(x_343, x_345); if (x_346 == 0) { x_262 = x_323; -x_263 = x_326; -x_264 = x_325; -x_265 = x_324; +x_263 = x_325; +x_264 = x_324; +x_265 = x_326; x_266 = x_327; x_267 = x_329; x_268 = x_328; -x_269 = x_332; +x_269 = x_330; x_270 = x_331; -x_271 = x_330; -x_272 = x_334; -x_273 = x_333; +x_271 = x_332; +x_272 = x_333; +x_273 = x_334; x_274 = x_335; x_275 = x_336; x_276 = x_337; @@ -57419,17 +57419,17 @@ x_350 = lean_ctor_get(x_349, 1); lean_inc(x_350); lean_dec(x_349); x_262 = x_323; -x_263 = x_326; -x_264 = x_325; -x_265 = x_324; +x_263 = x_325; +x_264 = x_324; +x_265 = x_326; x_266 = x_327; x_267 = x_329; x_268 = x_328; -x_269 = x_332; +x_269 = x_330; x_270 = x_331; -x_271 = x_330; -x_272 = x_334; -x_273 = x_333; +x_271 = x_332; +x_272 = x_333; +x_273 = x_334; x_274 = x_350; x_275 = x_336; x_276 = x_337; @@ -57449,10 +57449,10 @@ lean_dec(x_339); lean_dec_ref(x_338); lean_dec(x_337); lean_dec_ref(x_336); -lean_dec(x_333); -lean_dec_ref(x_332); +lean_dec_ref(x_334); +lean_dec_ref(x_333); lean_dec(x_331); -lean_dec_ref(x_330); +lean_dec(x_330); lean_dec_ref(x_329); lean_dec(x_328); lean_dec(x_327); @@ -58227,8 +58227,8 @@ lean_dec(x_364); x_503 = lean_ctor_get(x_484, 0); lean_inc(x_503); lean_dec_ref(x_484); -x_231 = x_503; -x_232 = x_450; +x_231 = x_450; +x_232 = x_503; x_233 = x_502; x_234 = x_356; x_235 = x_357; @@ -58273,8 +58273,8 @@ lean_dec_ref(x_512); x_514 = lean_ctor_get(x_513, 1); lean_inc(x_514); lean_dec(x_513); -x_231 = x_507; -x_232 = x_450; +x_231 = x_450; +x_232 = x_507; x_233 = x_514; x_234 = x_356; x_235 = x_357; @@ -58347,8 +58347,8 @@ lean_dec_ref(x_524); x_526 = lean_ctor_get(x_525, 1); lean_inc(x_526); lean_dec(x_525); -x_231 = x_518; -x_232 = x_450; +x_231 = x_450; +x_232 = x_518; x_233 = x_526; x_234 = x_356; x_235 = x_357; @@ -58494,18 +58494,18 @@ lean_dec(x_450); x_558 = lean_ctor_get(x_484, 0); lean_inc(x_558); lean_dec_ref(x_484); -x_323 = x_451; -x_324 = x_549; -x_325 = x_555; -x_326 = x_557; -x_327 = x_552; -x_328 = x_548; -x_329 = x_551; -x_330 = x_553; -x_331 = x_554; -x_332 = x_556; -x_333 = x_558; -x_334 = x_550; +x_323 = x_552; +x_324 = x_548; +x_325 = x_557; +x_326 = x_554; +x_327 = x_549; +x_328 = x_558; +x_329 = x_553; +x_330 = x_555; +x_331 = x_451; +x_332 = x_550; +x_333 = x_556; +x_334 = x_551; x_335 = x_547; x_336 = x_356; x_337 = x_357; @@ -58569,18 +58569,18 @@ lean_dec_ref(x_577); x_579 = lean_ctor_get(x_578, 1); lean_inc(x_579); lean_dec(x_578); -x_323 = x_451; -x_324 = x_563; -x_325 = x_569; -x_326 = x_571; -x_327 = x_566; -x_328 = x_562; -x_329 = x_565; -x_330 = x_567; -x_331 = x_568; -x_332 = x_570; -x_333 = x_572; -x_334 = x_564; +x_323 = x_566; +x_324 = x_562; +x_325 = x_571; +x_326 = x_568; +x_327 = x_563; +x_328 = x_572; +x_329 = x_567; +x_330 = x_569; +x_331 = x_451; +x_332 = x_564; +x_333 = x_570; +x_334 = x_565; x_335 = x_579; x_336 = x_356; x_337 = x_357; @@ -58681,18 +58681,18 @@ lean_dec_ref(x_599); x_601 = lean_ctor_get(x_600, 1); lean_inc(x_601); lean_dec(x_600); -x_323 = x_451; -x_324 = x_584; -x_325 = x_590; -x_326 = x_592; -x_327 = x_587; -x_328 = x_583; -x_329 = x_586; -x_330 = x_588; -x_331 = x_589; -x_332 = x_591; -x_333 = x_593; -x_334 = x_585; +x_323 = x_587; +x_324 = x_583; +x_325 = x_592; +x_326 = x_589; +x_327 = x_584; +x_328 = x_593; +x_329 = x_588; +x_330 = x_590; +x_331 = x_451; +x_332 = x_585; +x_333 = x_591; +x_334 = x_586; x_335 = x_601; x_336 = x_356; x_337 = x_357; @@ -61054,13 +61054,13 @@ goto block_17; { lean_object* x_34; lean_object* x_35; lean_object* x_36; x_34 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_34, 0, x_32); -x_35 = l_Lean_PersistentArray_set___redArg(x_30, x_33, x_34); +lean_ctor_set(x_34, 0, x_29); +x_35 = l_Lean_PersistentArray_set___redArg(x_28, x_33, x_34); lean_dec(x_33); x_36 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_36, 0, x_31); +lean_ctor_set(x_36, 0, x_30); lean_ctor_set(x_36, 1, x_35); -lean_ctor_set(x_36, 2, x_29); +lean_ctor_set(x_36, 2, x_32); x_24 = lean_box(0); x_25 = x_36; goto block_27; @@ -61068,14 +61068,14 @@ goto block_27; block_46: { lean_object* x_44; lean_object* x_45; -lean_inc_ref(x_42); -x_44 = l_Lean_PersistentHashMap_insert___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtorLCtx_spec__1___redArg(x_39, x_43, x_42); -x_45 = lean_ctor_get(x_42, 0); +lean_inc_ref(x_39); +x_44 = l_Lean_PersistentHashMap_insert___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtorLCtx_spec__1___redArg(x_40, x_43, x_39); +x_45 = lean_ctor_get(x_39, 0); lean_inc(x_45); -x_28 = lean_box(0); -x_29 = x_40; -x_30 = x_41; -x_31 = x_44; +x_28 = x_38; +x_29 = x_39; +x_30 = x_44; +x_31 = lean_box(0); x_32 = x_42; x_33 = x_45; goto block_37; @@ -61161,11 +61161,11 @@ x_76 = l_Lean_mkAppB(x_74, x_75, x_61); x_77 = l_Lean_LocalDecl_setType(x_70, x_76); x_78 = lean_ctor_get(x_77, 1); lean_inc(x_78); -x_38 = lean_box(0); -x_39 = x_66; -x_40 = x_68; -x_41 = x_67; -x_42 = x_77; +x_38 = x_67; +x_39 = x_77; +x_40 = x_66; +x_41 = lean_box(0); +x_42 = x_68; x_43 = x_78; goto block_46; } @@ -61682,13 +61682,13 @@ goto block_21; { lean_object* x_38; lean_object* x_39; lean_object* x_40; x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_35); -x_39 = l_Lean_PersistentArray_set___redArg(x_33, x_37, x_38); +lean_ctor_set(x_38, 0, x_34); +x_39 = l_Lean_PersistentArray_set___redArg(x_35, x_37, x_38); lean_dec(x_37); x_40 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_40, 0, x_36); lean_ctor_set(x_40, 1, x_39); -lean_ctor_set(x_40, 2, x_34); +lean_ctor_set(x_40, 2, x_32); x_28 = lean_box(0); x_29 = x_40; goto block_31; @@ -61696,14 +61696,14 @@ goto block_31; block_50: { lean_object* x_48; lean_object* x_49; -lean_inc_ref(x_45); -x_48 = l_Lean_PersistentHashMap_insert___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtorLCtx_spec__1___redArg(x_46, x_47, x_45); -x_49 = lean_ctor_get(x_45, 0); +lean_inc_ref(x_44); +x_48 = l_Lean_PersistentHashMap_insert___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtorLCtx_spec__1___redArg(x_45, x_47, x_44); +x_49 = lean_ctor_get(x_44, 0); lean_inc(x_49); -x_32 = lean_box(0); -x_33 = x_42; +x_32 = x_42; +x_33 = lean_box(0); x_34 = x_44; -x_35 = x_45; +x_35 = x_46; x_36 = x_48; x_37 = x_49; goto block_41; @@ -61789,11 +61789,11 @@ x_80 = l_Lean_mkAppB(x_78, x_79, x_65); x_81 = l_Lean_LocalDecl_setType(x_74, x_80); x_82 = lean_ctor_get(x_81, 1); lean_inc(x_82); -x_42 = x_71; +x_42 = x_72; x_43 = lean_box(0); -x_44 = x_72; -x_45 = x_81; -x_46 = x_70; +x_44 = x_81; +x_45 = x_70; +x_46 = x_71; x_47 = x_82; goto block_50; } @@ -65794,8 +65794,8 @@ goto block_170; block_102: { lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = lean_st_ref_get(x_35); -x_38 = lean_st_ref_take(x_35); +x_37 = lean_st_ref_get(x_29); +x_38 = lean_st_ref_take(x_29); x_39 = !lean_is_exclusive(x_38); if (x_39 == 0) { @@ -65804,7 +65804,7 @@ x_40 = lean_ctor_get(x_38, 1); lean_dec(x_40); x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__2___closed__2; lean_ctor_set(x_38, 1, x_41); -x_42 = lean_st_ref_set(x_35, x_38); +x_42 = lean_st_ref_set(x_29, x_38); x_43 = lean_ctor_get(x_37, 1); lean_inc_ref(x_43); lean_dec(x_37); @@ -65813,14 +65813,14 @@ x_45 = 0; x_46 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__0(x_44, x_45, x_36); x_47 = 1; x_48 = 0; -lean_inc_ref(x_29); -x_49 = l_Lean_LocalContext_mkForall(x_29, x_46, x_30, x_47, x_48); -lean_dec_ref(x_30); +lean_inc_ref(x_32); +x_49 = l_Lean_LocalContext_mkForall(x_32, x_46, x_35, x_47, x_48); +lean_dec_ref(x_35); lean_dec_ref(x_46); x_50 = lean_box(x_48); x_51 = lean_box(x_47); x_52 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__0___boxed), 15, 7); -lean_closure_set(x_52, 0, x_24); +lean_closure_set(x_52, 0, x_25); lean_closure_set(x_52, 1, x_5); lean_closure_set(x_52, 2, x_2); lean_closure_set(x_52, 3, x_50); @@ -65828,7 +65828,7 @@ lean_closure_set(x_52, 4, x_51); lean_closure_set(x_52, 5, x_23); lean_closure_set(x_52, 6, x_49); x_53 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__2___closed__3; -x_54 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_29, x_53, x_52, x_27, x_33, x_32, x_28, x_35, x_26, x_34); +x_54 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_32, x_53, x_52, x_31, x_30, x_34, x_27, x_29, x_26, x_28); if (lean_obj_tag(x_54) == 0) { uint8_t x_55; @@ -65839,9 +65839,9 @@ lean_object* x_56; lean_object* x_57; uint8_t x_58; x_56 = lean_ctor_get(x_54, 0); lean_inc(x_56); lean_ctor_set_tag(x_54, 1); -x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_25, x_43, x_54); +x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_24, x_43, x_54); lean_dec_ref(x_54); -lean_dec(x_25); +lean_dec(x_24); x_58 = !lean_is_exclusive(x_57); if (x_58 == 0) { @@ -65869,9 +65869,9 @@ lean_dec(x_54); lean_inc(x_61); x_62 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_62, 0, x_61); -x_63 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_25, x_43, x_62); +x_63 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_24, x_43, x_62); lean_dec_ref(x_62); -lean_dec(x_25); +lean_dec(x_24); if (lean_is_exclusive(x_63)) { lean_ctor_release(x_63, 0); x_64 = x_63; @@ -65895,8 +65895,8 @@ x_66 = lean_ctor_get(x_54, 0); lean_inc(x_66); lean_dec_ref(x_54); x_67 = lean_box(0); -x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_25, x_43, x_67); -lean_dec(x_25); +x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_24, x_43, x_67); +lean_dec(x_24); x_69 = !lean_is_exclusive(x_68); if (x_69 == 0) { @@ -65936,7 +65936,7 @@ lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_73); lean_ctor_set(x_77, 3, x_74); lean_ctor_set(x_77, 4, x_75); -x_78 = lean_st_ref_set(x_35, x_77); +x_78 = lean_st_ref_set(x_29, x_77); x_79 = lean_ctor_get(x_37, 1); lean_inc_ref(x_79); lean_dec(x_37); @@ -65945,14 +65945,14 @@ x_81 = 0; x_82 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__0(x_80, x_81, x_36); x_83 = 1; x_84 = 0; -lean_inc_ref(x_29); -x_85 = l_Lean_LocalContext_mkForall(x_29, x_82, x_30, x_83, x_84); -lean_dec_ref(x_30); +lean_inc_ref(x_32); +x_85 = l_Lean_LocalContext_mkForall(x_32, x_82, x_35, x_83, x_84); +lean_dec_ref(x_35); lean_dec_ref(x_82); x_86 = lean_box(x_84); x_87 = lean_box(x_83); x_88 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__0___boxed), 15, 7); -lean_closure_set(x_88, 0, x_24); +lean_closure_set(x_88, 0, x_25); lean_closure_set(x_88, 1, x_5); lean_closure_set(x_88, 2, x_2); lean_closure_set(x_88, 3, x_86); @@ -65960,7 +65960,7 @@ lean_closure_set(x_88, 4, x_87); lean_closure_set(x_88, 5, x_23); lean_closure_set(x_88, 6, x_85); x_89 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__2___closed__3; -x_90 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_29, x_89, x_88, x_27, x_33, x_32, x_28, x_35, x_26, x_34); +x_90 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_32, x_89, x_88, x_31, x_30, x_34, x_27, x_29, x_26, x_28); if (lean_obj_tag(x_90) == 0) { lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; @@ -65981,9 +65981,9 @@ if (lean_is_scalar(x_92)) { lean_ctor_set_tag(x_93, 1); } lean_ctor_set(x_93, 0, x_91); -x_94 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_25, x_79, x_93); +x_94 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_24, x_79, x_93); lean_dec_ref(x_93); -lean_dec(x_25); +lean_dec(x_24); if (lean_is_exclusive(x_94)) { lean_ctor_release(x_94, 0); x_95 = x_94; @@ -66006,8 +66006,8 @@ x_97 = lean_ctor_get(x_90, 0); lean_inc(x_97); lean_dec_ref(x_90); x_98 = lean_box(0); -x_99 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_25, x_79, x_98); -lean_dec(x_25); +x_99 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_24, x_79, x_98); +lean_dec(x_24); if (lean_is_exclusive(x_99)) { lean_ctor_release(x_99, 0); x_100 = x_99; @@ -66068,18 +66068,18 @@ x_126 = lean_nat_dec_lt(x_123, x_124); if (x_126 == 0) { lean_inc(x_108); -x_24 = x_103; -x_25 = x_108; +x_24 = x_108; +x_25 = x_103; x_26 = x_109; -x_27 = x_120; -x_28 = x_107; -x_29 = x_114; -x_30 = x_121; -x_31 = lean_box(0); -x_32 = x_106; -x_33 = x_105; -x_34 = x_110; -x_35 = x_108; +x_27 = x_107; +x_28 = x_110; +x_29 = x_108; +x_30 = x_105; +x_31 = x_120; +x_32 = x_114; +x_33 = lean_box(0); +x_34 = x_106; +x_35 = x_121; x_36 = x_125; goto block_102; } @@ -66090,18 +66090,18 @@ x_127 = lean_nat_dec_le(x_124, x_124); if (x_127 == 0) { lean_inc(x_108); -x_24 = x_103; -x_25 = x_108; +x_24 = x_108; +x_25 = x_103; x_26 = x_109; -x_27 = x_120; -x_28 = x_107; -x_29 = x_114; -x_30 = x_121; -x_31 = lean_box(0); -x_32 = x_106; -x_33 = x_105; -x_34 = x_110; -x_35 = x_108; +x_27 = x_107; +x_28 = x_110; +x_29 = x_108; +x_30 = x_105; +x_31 = x_120; +x_32 = x_114; +x_33 = lean_box(0); +x_34 = x_106; +x_35 = x_121; x_36 = x_125; goto block_102; } @@ -66112,18 +66112,18 @@ x_128 = 0; x_129 = lean_usize_of_nat(x_124); x_130 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__3(x_122, x_128, x_129, x_125); lean_inc(x_108); -x_24 = x_103; -x_25 = x_108; +x_24 = x_108; +x_25 = x_103; x_26 = x_109; -x_27 = x_120; -x_28 = x_107; -x_29 = x_114; -x_30 = x_121; -x_31 = lean_box(0); -x_32 = x_106; -x_33 = x_105; -x_34 = x_110; -x_35 = x_108; +x_27 = x_107; +x_28 = x_110; +x_29 = x_108; +x_30 = x_105; +x_31 = x_120; +x_32 = x_114; +x_33 = lean_box(0); +x_34 = x_106; +x_35 = x_121; x_36 = x_130; goto block_102; } @@ -66483,8 +66483,8 @@ goto block_311; block_253: { 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; size_t x_231; size_t x_232; lean_object* x_233; uint8_t x_234; uint8_t 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_220 = lean_st_ref_get(x_218); -x_221 = lean_st_ref_take(x_218); +x_220 = lean_st_ref_get(x_212); +x_221 = lean_st_ref_take(x_212); x_222 = lean_ctor_get(x_221, 0); lean_inc_ref(x_222); x_223 = lean_ctor_get(x_221, 2); @@ -66515,7 +66515,7 @@ lean_ctor_set(x_228, 1, x_227); lean_ctor_set(x_228, 2, x_223); lean_ctor_set(x_228, 3, x_224); lean_ctor_set(x_228, 4, x_225); -x_229 = lean_st_ref_set(x_218, x_228); +x_229 = lean_st_ref_set(x_212, x_228); x_230 = lean_ctor_get(x_220, 1); lean_inc_ref(x_230); lean_dec(x_220); @@ -66524,14 +66524,14 @@ x_232 = 0; x_233 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__0(x_231, x_232, x_219); x_234 = 1; x_235 = 0; -lean_inc_ref(x_212); -x_236 = l_Lean_LocalContext_mkForall(x_212, x_233, x_213, x_234, x_235); -lean_dec_ref(x_213); +lean_inc_ref(x_215); +x_236 = l_Lean_LocalContext_mkForall(x_215, x_233, x_218, x_234, x_235); +lean_dec_ref(x_218); lean_dec_ref(x_233); x_237 = lean_box(x_235); x_238 = lean_box(x_234); x_239 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__0___boxed), 15, 7); -lean_closure_set(x_239, 0, x_207); +lean_closure_set(x_239, 0, x_208); lean_closure_set(x_239, 1, x_5); lean_closure_set(x_239, 2, x_2); lean_closure_set(x_239, 3, x_237); @@ -66539,7 +66539,7 @@ lean_closure_set(x_239, 4, x_238); lean_closure_set(x_239, 5, x_206); lean_closure_set(x_239, 6, x_236); x_240 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__2___closed__3; -x_241 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_212, x_240, x_239, x_210, x_216, x_215, x_211, x_218, x_209, x_217); +x_241 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_215, x_240, x_239, x_214, x_213, x_217, x_210, x_212, x_209, x_211); if (lean_obj_tag(x_241) == 0) { lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; @@ -66560,9 +66560,9 @@ if (lean_is_scalar(x_243)) { lean_ctor_set_tag(x_244, 1); } lean_ctor_set(x_244, 0, x_242); -x_245 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_208, x_230, x_244); +x_245 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_207, x_230, x_244); lean_dec_ref(x_244); -lean_dec(x_208); +lean_dec(x_207); if (lean_is_exclusive(x_245)) { lean_ctor_release(x_245, 0); x_246 = x_245; @@ -66585,8 +66585,8 @@ x_248 = lean_ctor_get(x_241, 0); lean_inc(x_248); lean_dec_ref(x_241); x_249 = lean_box(0); -x_250 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_208, x_230, x_249); -lean_dec(x_208); +x_250 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor___lam__1(x_207, x_230, x_249); +lean_dec(x_207); if (lean_is_exclusive(x_250)) { lean_ctor_release(x_250, 0); x_251 = x_250; @@ -66646,18 +66646,18 @@ x_277 = lean_nat_dec_lt(x_274, x_275); if (x_277 == 0) { lean_inc(x_259); -x_207 = x_254; -x_208 = x_259; +x_207 = x_259; +x_208 = x_254; x_209 = x_260; -x_210 = x_271; -x_211 = x_258; -x_212 = x_265; -x_213 = x_272; -x_214 = lean_box(0); -x_215 = x_257; -x_216 = x_256; -x_217 = x_261; -x_218 = x_259; +x_210 = x_258; +x_211 = x_261; +x_212 = x_259; +x_213 = x_256; +x_214 = x_271; +x_215 = x_265; +x_216 = lean_box(0); +x_217 = x_257; +x_218 = x_272; x_219 = x_276; goto block_253; } @@ -66668,18 +66668,18 @@ x_278 = lean_nat_dec_le(x_275, x_275); if (x_278 == 0) { lean_inc(x_259); -x_207 = x_254; -x_208 = x_259; +x_207 = x_259; +x_208 = x_254; x_209 = x_260; -x_210 = x_271; -x_211 = x_258; -x_212 = x_265; -x_213 = x_272; -x_214 = lean_box(0); -x_215 = x_257; -x_216 = x_256; -x_217 = x_261; -x_218 = x_259; +x_210 = x_258; +x_211 = x_261; +x_212 = x_259; +x_213 = x_256; +x_214 = x_271; +x_215 = x_265; +x_216 = lean_box(0); +x_217 = x_257; +x_218 = x_272; x_219 = x_276; goto block_253; } @@ -66690,18 +66690,18 @@ x_279 = 0; x_280 = lean_usize_of_nat(x_275); x_281 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__3(x_273, x_279, x_280, x_276); lean_inc(x_259); -x_207 = x_254; -x_208 = x_259; +x_207 = x_259; +x_208 = x_254; x_209 = x_260; -x_210 = x_271; -x_211 = x_258; -x_212 = x_265; -x_213 = x_272; -x_214 = lean_box(0); -x_215 = x_257; -x_216 = x_256; -x_217 = x_261; -x_218 = x_259; +x_210 = x_258; +x_211 = x_261; +x_212 = x_259; +x_213 = x_256; +x_214 = x_271; +x_215 = x_265; +x_216 = lean_box(0); +x_217 = x_257; +x_218 = x_272; x_219 = x_281; goto block_253; } @@ -67590,9 +67590,9 @@ x_51 = lean_nat_dec_lt(x_44, x_50); if (x_51 == 0) { lean_dec_ref(x_49); -lean_dec_ref(x_47); -x_13 = x_46; -x_14 = x_48; +lean_dec_ref(x_48); +x_13 = x_47; +x_14 = x_45; x_15 = lean_box(0); goto block_30; } @@ -67605,7 +67605,7 @@ lean_inc_ref(x_10); lean_inc(x_9); lean_inc_ref(x_8); lean_inc_ref(x_4); -x_53 = l___private_Init_Data_Array_Basic_0__Array_foldrMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtorExpr_spec__2___redArg(x_47, x_4, x_49, x_52, x_39, x_46, x_48, x_8, x_9, x_10, x_11); +x_53 = l___private_Init_Data_Array_Basic_0__Array_foldrMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtorExpr_spec__2___redArg(x_48, x_4, x_49, x_52, x_39, x_47, x_45, x_8, x_9, x_10, x_11); lean_dec_ref(x_49); if (lean_obj_tag(x_53) == 0) { @@ -67667,10 +67667,10 @@ x_69 = lean_nat_dec_lt(x_44, x_58); if (x_69 == 0) { lean_dec_ref(x_33); -x_45 = lean_box(0); -x_46 = x_67; -x_47 = x_65; -x_48 = x_63; +x_45 = x_63; +x_46 = lean_box(0); +x_47 = x_67; +x_48 = x_65; x_49 = x_68; goto block_57; } @@ -67681,10 +67681,10 @@ x_70 = lean_nat_dec_le(x_58, x_58); if (x_70 == 0) { lean_dec_ref(x_33); -x_45 = lean_box(0); -x_46 = x_67; -x_47 = x_65; -x_48 = x_63; +x_45 = x_63; +x_46 = lean_box(0); +x_47 = x_67; +x_48 = x_65; x_49 = x_68; goto block_57; } @@ -67694,10 +67694,10 @@ size_t x_71; lean_object* x_72; x_71 = lean_usize_of_nat(x_58); x_72 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtorExpr_spec__3(x_33, x_39, x_71, x_68); lean_dec_ref(x_33); -x_45 = lean_box(0); -x_46 = x_67; -x_47 = x_65; -x_48 = x_63; +x_45 = x_63; +x_46 = lean_box(0); +x_47 = x_67; +x_48 = x_65; x_49 = x_72; goto block_57; } @@ -71730,24 +71730,24 @@ return x_8; block_21: { uint8_t x_17; -x_17 = lean_nat_dec_lt(x_15, x_16); +x_17 = lean_nat_dec_lt(x_14, x_16); if (x_17 == 0) { lean_dec(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); +lean_dec_ref(x_15); +lean_dec(x_14); x_9 = x_7; goto block_13; } else { size_t x_18; size_t x_19; uint8_t x_20; -x_18 = lean_usize_of_nat(x_15); -lean_dec(x_15); +x_18 = lean_usize_of_nat(x_14); +lean_dec(x_14); x_19 = lean_usize_of_nat(x_16); lean_dec(x_16); -x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_14, x_18, x_19); -lean_dec_ref(x_14); +x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_15, x_18, x_19); +lean_dec_ref(x_15); if (x_20 == 0) { x_9 = x_20; @@ -71788,15 +71788,15 @@ x_31 = lean_nat_dec_le(x_28, x_30); if (x_31 == 0) { lean_dec(x_28); -x_14 = x_26; -x_15 = x_27; +x_14 = x_27; +x_15 = x_26; x_16 = x_30; goto block_21; } else { -x_14 = x_26; -x_15 = x_27; +x_14 = x_27; +x_15 = x_26; x_16 = x_28; goto block_21; } @@ -71857,24 +71857,24 @@ return x_8; block_21: { uint8_t x_17; -x_17 = lean_nat_dec_lt(x_15, x_16); +x_17 = lean_nat_dec_lt(x_14, x_16); if (x_17 == 0) { lean_dec(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); +lean_dec_ref(x_15); +lean_dec(x_14); x_9 = x_7; goto block_13; } else { size_t x_18; size_t x_19; uint8_t x_20; -x_18 = lean_usize_of_nat(x_15); -lean_dec(x_15); +x_18 = lean_usize_of_nat(x_14); +lean_dec(x_14); x_19 = lean_usize_of_nat(x_16); lean_dec(x_16); -x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_14, x_18, x_19); -lean_dec_ref(x_14); +x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_15, x_18, x_19); +lean_dec_ref(x_15); if (x_20 == 0) { x_9 = x_20; @@ -71915,15 +71915,15 @@ x_31 = lean_nat_dec_le(x_28, x_30); if (x_31 == 0) { lean_dec(x_28); -x_14 = x_26; -x_15 = x_27; +x_14 = x_27; +x_15 = x_26; x_16 = x_30; goto block_21; } else { -x_14 = x_26; -x_15 = x_27; +x_14 = x_27; +x_15 = x_26; x_16 = x_28; goto block_21; } @@ -71984,24 +71984,24 @@ return x_7; block_20: { uint8_t x_16; -x_16 = lean_nat_dec_lt(x_13, x_15); +x_16 = lean_nat_dec_lt(x_14, x_15); if (x_16 == 0) { lean_dec(x_15); -lean_dec_ref(x_14); -lean_dec(x_13); +lean_dec(x_14); +lean_dec_ref(x_13); x_8 = x_6; goto block_12; } else { size_t x_17; size_t x_18; uint8_t x_19; -x_17 = lean_usize_of_nat(x_13); -lean_dec(x_13); +x_17 = lean_usize_of_nat(x_14); +lean_dec(x_14); x_18 = lean_usize_of_nat(x_15); lean_dec(x_15); -x_19 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_14, x_17, x_18); -lean_dec_ref(x_14); +x_19 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_13, x_17, x_18); +lean_dec_ref(x_13); x_8 = x_19; goto block_12; } @@ -72034,15 +72034,15 @@ x_30 = lean_nat_dec_le(x_27, x_29); if (x_30 == 0) { lean_dec(x_27); -x_13 = x_26; -x_14 = x_25; +x_13 = x_25; +x_14 = x_26; x_15 = x_29; goto block_20; } else { -x_13 = x_26; -x_14 = x_25; +x_13 = x_25; +x_14 = x_26; x_15 = x_27; goto block_20; } @@ -72207,7 +72207,7 @@ return x_54; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; uint8_t x_79; uint8_t x_90; lean_object* x_91; +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_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; uint8_t x_79; uint8_t x_90; lean_object* x_91; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -72277,11 +72277,11 @@ goto block_51; block_78: { uint8_t x_74; -x_74 = lean_nat_dec_lt(x_72, x_73); +x_74 = lean_nat_dec_lt(x_71, x_73); if (x_74 == 0) { lean_dec(x_73); -lean_dec(x_72); +lean_dec(x_71); lean_dec_ref(x_70); lean_dec_ref(x_59); goto block_69; @@ -72289,12 +72289,12 @@ goto block_69; else { size_t x_75; size_t x_76; uint8_t x_77; -x_75 = lean_usize_of_nat(x_72); -lean_dec(x_72); +x_75 = lean_usize_of_nat(x_71); +lean_dec(x_71); x_76 = lean_usize_of_nat(x_73); lean_dec(x_73); lean_inc(x_6); -x_77 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_61, x_6, x_71, x_70, x_75, x_76); +x_77 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_61, x_6, x_72, x_70, x_75, x_76); lean_dec_ref(x_70); if (x_77 == 0) { @@ -72341,16 +72341,16 @@ if (x_88 == 0) { lean_dec(x_85); x_70 = x_83; -x_71 = x_79; -x_72 = x_84; +x_71 = x_84; +x_72 = x_79; x_73 = x_87; goto block_78; } else { x_70 = x_83; -x_71 = x_79; -x_72 = x_84; +x_71 = x_84; +x_72 = x_79; x_73 = x_85; goto block_78; } @@ -72654,7 +72654,7 @@ return x_54; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_79; uint8_t x_90; lean_object* x_91; +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_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; uint8_t x_79; uint8_t x_90; lean_object* x_91; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -72724,24 +72724,24 @@ goto block_51; block_78: { uint8_t x_74; -x_74 = lean_nat_dec_lt(x_71, x_73); +x_74 = lean_nat_dec_lt(x_70, x_73); if (x_74 == 0) { lean_dec(x_73); lean_dec_ref(x_72); -lean_dec(x_71); +lean_dec(x_70); lean_dec_ref(x_59); goto block_69; } else { size_t x_75; size_t x_76; uint8_t x_77; -x_75 = lean_usize_of_nat(x_71); -lean_dec(x_71); +x_75 = lean_usize_of_nat(x_70); +lean_dec(x_70); x_76 = lean_usize_of_nat(x_73); lean_dec(x_73); lean_inc(x_6); -x_77 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_61, x_6, x_70, x_72, x_75, x_76); +x_77 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_61, x_6, x_71, x_72, x_75, x_76); lean_dec_ref(x_72); if (x_77 == 0) { @@ -72787,16 +72787,16 @@ x_88 = lean_nat_dec_le(x_85, x_87); if (x_88 == 0) { lean_dec(x_85); -x_70 = x_79; -x_71 = x_84; +x_70 = x_84; +x_71 = x_79; x_72 = x_83; x_73 = x_87; goto block_78; } else { -x_70 = x_79; -x_71 = x_84; +x_70 = x_84; +x_71 = x_79; x_72 = x_83; x_73 = x_85; goto block_78; @@ -73965,7 +73965,7 @@ lean_ctor_set(x_54, 9, x_34); lean_ctor_set(x_54, 10, x_46); lean_ctor_set(x_54, 11, x_53); lean_ctor_set_uint8(x_54, sizeof(void*)*12, x_29); -x_55 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_54, x_51, x_47, x_48, x_49, x_52); +x_55 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_54, x_52, x_51, x_47, x_50, x_49); if (lean_obj_tag(x_55) == 0) { lean_object* x_56; lean_object* x_57; @@ -73992,12 +73992,12 @@ x_65 = lean_array_get_size(x_46); x_66 = lean_nat_dec_lt(x_44, x_65); if (x_66 == 0) { -x_47 = x_60; -x_48 = x_61; -x_49 = x_62; -x_50 = lean_box(0); -x_51 = x_59; -x_52 = x_63; +x_47 = x_61; +x_48 = lean_box(0); +x_49 = x_63; +x_50 = x_62; +x_51 = x_60; +x_52 = x_59; x_53 = x_24; goto block_58; } @@ -74010,12 +74010,12 @@ lean_inc(x_68); lean_dec(x_67); x_69 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_69, 0, x_68); -x_47 = x_60; -x_48 = x_61; -x_49 = x_62; -x_50 = lean_box(0); -x_51 = x_59; -x_52 = x_63; +x_47 = x_61; +x_48 = lean_box(0); +x_49 = x_63; +x_50 = x_62; +x_51 = x_60; +x_52 = x_59; x_53 = x_69; goto block_58; } @@ -74118,7 +74118,7 @@ lean_ctor_set(x_94, 9, x_34); lean_ctor_set(x_94, 10, x_86); lean_ctor_set(x_94, 11, x_93); lean_ctor_set_uint8(x_94, sizeof(void*)*12, x_29); -x_95 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_94, x_91, x_87, x_88, x_89, x_92); +x_95 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_94, x_92, x_91, x_87, x_90, x_89); if (lean_obj_tag(x_95) == 0) { lean_object* x_96; lean_object* x_97; @@ -74145,12 +74145,12 @@ x_105 = lean_array_get_size(x_86); x_106 = lean_nat_dec_lt(x_84, x_105); if (x_106 == 0) { -x_87 = x_100; -x_88 = x_101; -x_89 = x_102; -x_90 = lean_box(0); -x_91 = x_99; -x_92 = x_103; +x_87 = x_101; +x_88 = lean_box(0); +x_89 = x_103; +x_90 = x_102; +x_91 = x_100; +x_92 = x_99; x_93 = x_24; goto block_98; } @@ -74163,12 +74163,12 @@ lean_inc(x_108); lean_dec(x_107); x_109 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_109, 0, x_108); -x_87 = x_100; -x_88 = x_101; -x_89 = x_102; -x_90 = lean_box(0); -x_91 = x_99; -x_92 = x_103; +x_87 = x_101; +x_88 = lean_box(0); +x_89 = x_103; +x_90 = x_102; +x_91 = x_100; +x_92 = x_99; x_93 = x_109; goto block_98; } @@ -74511,7 +74511,7 @@ lean_ctor_set(x_56, 9, x_36); lean_ctor_set(x_56, 10, x_48); lean_ctor_set(x_56, 11, x_55); lean_ctor_set_uint8(x_56, sizeof(void*)*12, x_31); -x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_56, x_50, x_52, x_54, x_53, x_51); +x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_56, x_51, x_50, x_49, x_53, x_52); if (lean_obj_tag(x_57) == 0) { lean_object* x_58; lean_object* x_59; @@ -74538,12 +74538,12 @@ x_67 = lean_array_get_size(x_48); x_68 = lean_nat_dec_lt(x_46, x_67); if (x_68 == 0) { -x_49 = lean_box(0); -x_50 = x_61; -x_51 = x_65; -x_52 = x_62; +x_49 = x_63; +x_50 = x_62; +x_51 = x_61; +x_52 = x_65; x_53 = x_64; -x_54 = x_63; +x_54 = lean_box(0); x_55 = x_26; goto block_60; } @@ -74556,12 +74556,12 @@ lean_inc(x_70); lean_dec(x_69); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); -x_49 = lean_box(0); -x_50 = x_61; -x_51 = x_65; -x_52 = x_62; +x_49 = x_63; +x_50 = x_62; +x_51 = x_61; +x_52 = x_65; x_53 = x_64; -x_54 = x_63; +x_54 = lean_box(0); x_55 = x_71; goto block_60; } @@ -74664,7 +74664,7 @@ lean_ctor_set(x_96, 9, x_36); lean_ctor_set(x_96, 10, x_88); lean_ctor_set(x_96, 11, x_95); lean_ctor_set_uint8(x_96, sizeof(void*)*12, x_31); -x_97 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_96, x_90, x_92, x_94, x_93, x_91); +x_97 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_replaceFieldInfo___redArg(x_96, x_91, x_90, x_89, x_93, x_92); if (lean_obj_tag(x_97) == 0) { lean_object* x_98; lean_object* x_99; @@ -74691,12 +74691,12 @@ x_107 = lean_array_get_size(x_88); x_108 = lean_nat_dec_lt(x_86, x_107); if (x_108 == 0) { -x_89 = lean_box(0); -x_90 = x_101; -x_91 = x_105; -x_92 = x_102; +x_89 = x_103; +x_90 = x_102; +x_91 = x_101; +x_92 = x_105; x_93 = x_104; -x_94 = x_103; +x_94 = lean_box(0); x_95 = x_26; goto block_100; } @@ -74709,12 +74709,12 @@ lean_inc(x_110); lean_dec(x_109); x_111 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_111, 0, x_110); -x_89 = lean_box(0); -x_90 = x_101; -x_91 = x_105; -x_92 = x_102; +x_89 = x_103; +x_90 = x_102; +x_91 = x_101; +x_92 = x_105; x_93 = x_104; -x_94 = x_103; +x_94 = lean_box(0); x_95 = x_111; goto block_100; } @@ -76038,12 +76038,12 @@ goto block_32; block_22: { uint8_t x_17; -x_17 = lean_nat_dec_lt(x_14, x_16); +x_17 = lean_nat_dec_lt(x_15, x_16); if (x_17 == 0) { lean_dec(x_16); -lean_dec_ref(x_15); -lean_dec(x_14); +lean_dec(x_15); +lean_dec_ref(x_14); lean_dec(x_13); x_7 = x_6; goto block_11; @@ -76051,12 +76051,12 @@ goto block_11; else { size_t x_18; size_t x_19; uint8_t x_20; -x_18 = lean_usize_of_nat(x_14); -lean_dec(x_14); +x_18 = lean_usize_of_nat(x_15); +lean_dec(x_15); x_19 = lean_usize_of_nat(x_16); lean_dec(x_16); -x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_15, x_18, x_19); -lean_dec_ref(x_15); +x_20 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__14(x_1, x_14, x_18, x_19); +lean_dec_ref(x_14); if (x_20 == 0) { lean_dec(x_13); @@ -76102,15 +76102,15 @@ x_31 = lean_nat_dec_le(x_28, x_30); if (x_31 == 0) { lean_dec(x_28); -x_14 = x_27; -x_15 = x_26; +x_14 = x_26; +x_15 = x_27; x_16 = x_30; goto block_22; } else { -x_14 = x_27; -x_15 = x_26; +x_14 = x_26; +x_15 = x_27; x_16 = x_28; goto block_22; } @@ -76247,8 +76247,8 @@ goto block_30; block_60: { lean_object* x_59; -lean_dec(x_57); -x_59 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_56, x_55, x_58); +lean_dec(x_56); +x_59 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_57, x_55, x_58); lean_dec(x_58); x_44 = x_59; goto block_54; @@ -76256,13 +76256,13 @@ goto block_54; block_66: { uint8_t x_65; -x_65 = lean_nat_dec_le(x_64, x_62); +x_65 = lean_nat_dec_le(x_64, x_61); if (x_65 == 0) { -lean_dec(x_62); +lean_dec(x_61); lean_inc(x_64); x_55 = x_64; -x_56 = x_61; +x_56 = x_62; x_57 = x_63; x_58 = x_64; goto block_60; @@ -76270,9 +76270,9 @@ goto block_60; else { x_55 = x_64; -x_56 = x_61; +x_56 = x_62; x_57 = x_63; -x_58 = x_62; +x_58 = x_61; goto block_60; } } @@ -76293,18 +76293,18 @@ x_75 = lean_nat_dec_le(x_1, x_74); if (x_75 == 0) { lean_inc(x_74); -x_61 = x_70; -x_62 = x_74; -x_63 = x_71; +x_61 = x_74; +x_62 = x_71; +x_63 = x_70; x_64 = x_74; goto block_66; } else { lean_inc(x_1); -x_61 = x_70; -x_62 = x_74; -x_63 = x_71; +x_61 = x_74; +x_62 = x_71; +x_63 = x_70; x_64 = x_1; goto block_66; } @@ -76475,8 +76475,8 @@ goto block_30; block_117: { lean_object* x_116; -lean_dec(x_114); -x_116 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_113, x_112, x_115); +lean_dec(x_113); +x_116 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_114, x_112, x_115); lean_dec(x_115); x_101 = x_116; goto block_111; @@ -76484,13 +76484,13 @@ goto block_111; block_123: { uint8_t x_122; -x_122 = lean_nat_dec_le(x_121, x_119); +x_122 = lean_nat_dec_le(x_121, x_118); if (x_122 == 0) { -lean_dec(x_119); +lean_dec(x_118); lean_inc(x_121); x_112 = x_121; -x_113 = x_118; +x_113 = x_119; x_114 = x_120; x_115 = x_121; goto block_117; @@ -76498,9 +76498,9 @@ goto block_117; else { x_112 = x_121; -x_113 = x_118; +x_113 = x_119; x_114 = x_120; -x_115 = x_119; +x_115 = x_118; goto block_117; } } @@ -76521,18 +76521,18 @@ x_132 = lean_nat_dec_le(x_1, x_131); if (x_132 == 0) { lean_inc(x_131); -x_118 = x_127; -x_119 = x_131; -x_120 = x_128; +x_118 = x_131; +x_119 = x_128; +x_120 = x_127; x_121 = x_131; goto block_123; } else { lean_inc(x_1); -x_118 = x_127; -x_119 = x_131; -x_120 = x_128; +x_118 = x_131; +x_119 = x_128; +x_120 = x_127; x_121 = x_1; goto block_123; } @@ -76721,8 +76721,8 @@ goto block_30; block_177: { lean_object* x_176; -lean_dec(x_174); -x_176 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_173, x_172, x_175); +lean_dec(x_173); +x_176 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_174, x_172, x_175); lean_dec(x_175); x_161 = x_176; goto block_171; @@ -76730,13 +76730,13 @@ goto block_171; block_183: { uint8_t x_182; -x_182 = lean_nat_dec_le(x_181, x_179); +x_182 = lean_nat_dec_le(x_181, x_178); if (x_182 == 0) { -lean_dec(x_179); +lean_dec(x_178); lean_inc(x_181); x_172 = x_181; -x_173 = x_178; +x_173 = x_179; x_174 = x_180; x_175 = x_181; goto block_177; @@ -76744,9 +76744,9 @@ goto block_177; else { x_172 = x_181; -x_173 = x_178; +x_173 = x_179; x_174 = x_180; -x_175 = x_179; +x_175 = x_178; goto block_177; } } @@ -76767,18 +76767,18 @@ x_192 = lean_nat_dec_le(x_1, x_191); if (x_192 == 0) { lean_inc(x_191); -x_178 = x_187; -x_179 = x_191; -x_180 = x_188; +x_178 = x_191; +x_179 = x_188; +x_180 = x_187; x_181 = x_191; goto block_183; } else { lean_inc(x_1); -x_178 = x_187; -x_179 = x_191; -x_180 = x_188; +x_178 = x_191; +x_179 = x_188; +x_180 = x_187; x_181 = x_1; goto block_183; } @@ -78734,7 +78734,7 @@ return x_10; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addDefaults_spec__2_spec__2___lam__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_117; +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; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_117; x_117 = l_Lean_instantiateMVars___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_reduceFieldProjs_spec__2___redArg(x_9, x_10, x_14); if (lean_obj_tag(x_117) == 0) { @@ -79004,8 +79004,8 @@ return x_153; lean_object* x_26; lean_inc(x_24); lean_inc_ref(x_23); -lean_inc_ref(x_19); -x_26 = lean_infer_type(x_19, x_21, x_22, x_23, x_24); +lean_inc_ref(x_18); +x_26 = lean_infer_type(x_18, x_21, x_22, x_23, x_24); if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_object* x_28; lean_object* x_29; @@ -79013,7 +79013,7 @@ x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); lean_dec_ref(x_26); x_28 = lean_box(1); -x_29 = l_Lean_mkDefinitionValInferringUnsafe___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtor_spec__0___redArg(x_8, x_1, x_27, x_19, x_28, x_20, x_24); +x_29 = l_Lean_mkDefinitionValInferringUnsafe___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtor_spec__0___redArg(x_8, x_1, x_27, x_18, x_28, x_20, x_24); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; uint8_t x_31; @@ -79028,7 +79028,7 @@ x_32 = lean_ctor_get(x_30, 0); x_33 = lean_ctor_get(x_30, 1); x_34 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_34, 0, x_32); -x_35 = l_Lean_addDecl(x_34, x_18, x_23, x_24); +x_35 = l_Lean_addDecl(x_34, x_19, x_23, x_24); if (lean_obj_tag(x_35) == 0) { uint8_t x_36; @@ -79085,7 +79085,7 @@ lean_inc(x_43); lean_dec(x_30); x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_43); -x_46 = l_Lean_addDecl(x_45, x_18, x_23, x_24); +x_46 = l_Lean_addDecl(x_45, x_19, x_23, x_24); if (lean_obj_tag(x_46) == 0) { lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; @@ -79160,7 +79160,7 @@ uint8_t x_57; lean_dec(x_24); lean_dec_ref(x_23); lean_dec_ref(x_20); -lean_dec_ref(x_19); +lean_dec_ref(x_18); lean_dec(x_8); lean_dec(x_1); x_57 = !lean_is_exclusive(x_26); @@ -79270,8 +79270,8 @@ lean_free_object(x_85); lean_dec_ref(x_80); lean_dec(x_12); lean_dec_ref(x_11); -x_18 = x_61; -x_19 = x_73; +x_18 = x_73; +x_19 = x_61; x_20 = x_87; x_21 = x_13; x_22 = x_14; @@ -79306,8 +79306,8 @@ lean_dec_ref(x_94); x_96 = lean_ctor_get(x_95, 1); lean_inc(x_96); lean_dec(x_95); -x_18 = x_61; -x_19 = x_73; +x_18 = x_73; +x_19 = x_61; x_20 = x_96; x_21 = x_13; x_22 = x_14; @@ -79341,8 +79341,8 @@ if (x_98 == 0) lean_dec_ref(x_80); lean_dec(x_12); lean_dec_ref(x_11); -x_18 = x_61; -x_19 = x_73; +x_18 = x_73; +x_19 = x_61; x_20 = x_97; x_21 = x_13; x_22 = x_14; @@ -79377,8 +79377,8 @@ lean_dec_ref(x_104); x_106 = lean_ctor_get(x_105, 1); lean_inc(x_106); lean_dec(x_105); -x_18 = x_61; -x_19 = x_73; +x_18 = x_73; +x_19 = x_61; x_20 = x_106; x_21 = x_13; x_22 = x_14; @@ -79790,7 +79790,7 @@ goto _start; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addDefaults_spec__2___redArg___lam__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -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; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_117; +uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_117; x_117 = l_Lean_instantiateMVars___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_reduceFieldProjs_spec__2___redArg(x_9, x_10, x_14); if (lean_obj_tag(x_117) == 0) { @@ -80060,8 +80060,8 @@ return x_153; lean_object* x_26; lean_inc(x_24); lean_inc_ref(x_23); -lean_inc_ref(x_18); -x_26 = lean_infer_type(x_18, x_21, x_22, x_23, x_24); +lean_inc_ref(x_19); +x_26 = lean_infer_type(x_19, x_21, x_22, x_23, x_24); if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_object* x_28; lean_object* x_29; @@ -80069,7 +80069,7 @@ x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); lean_dec_ref(x_26); x_28 = lean_box(1); -x_29 = l_Lean_mkDefinitionValInferringUnsafe___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtor_spec__0___redArg(x_8, x_1, x_27, x_18, x_28, x_20, x_24); +x_29 = l_Lean_mkDefinitionValInferringUnsafe___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtor_spec__0___redArg(x_8, x_1, x_27, x_19, x_28, x_20, x_24); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; uint8_t x_31; @@ -80084,7 +80084,7 @@ x_32 = lean_ctor_get(x_30, 0); x_33 = lean_ctor_get(x_30, 1); x_34 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_34, 0, x_32); -x_35 = l_Lean_addDecl(x_34, x_19, x_23, x_24); +x_35 = l_Lean_addDecl(x_34, x_18, x_23, x_24); if (lean_obj_tag(x_35) == 0) { uint8_t x_36; @@ -80141,7 +80141,7 @@ lean_inc(x_43); lean_dec(x_30); x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_43); -x_46 = l_Lean_addDecl(x_45, x_19, x_23, x_24); +x_46 = l_Lean_addDecl(x_45, x_18, x_23, x_24); if (lean_obj_tag(x_46) == 0) { lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; @@ -80216,7 +80216,7 @@ uint8_t x_57; lean_dec(x_24); lean_dec_ref(x_23); lean_dec_ref(x_20); -lean_dec_ref(x_18); +lean_dec_ref(x_19); lean_dec(x_8); lean_dec(x_1); x_57 = !lean_is_exclusive(x_26); @@ -80326,8 +80326,8 @@ lean_free_object(x_85); lean_dec_ref(x_80); lean_dec(x_12); lean_dec_ref(x_11); -x_18 = x_73; -x_19 = x_61; +x_18 = x_61; +x_19 = x_73; x_20 = x_87; x_21 = x_13; x_22 = x_14; @@ -80362,8 +80362,8 @@ lean_dec_ref(x_94); x_96 = lean_ctor_get(x_95, 1); lean_inc(x_96); lean_dec(x_95); -x_18 = x_73; -x_19 = x_61; +x_18 = x_61; +x_19 = x_73; x_20 = x_96; x_21 = x_13; x_22 = x_14; @@ -80397,8 +80397,8 @@ if (x_98 == 0) lean_dec_ref(x_80); lean_dec(x_12); lean_dec_ref(x_11); -x_18 = x_73; -x_19 = x_61; +x_18 = x_61; +x_19 = x_73; x_20 = x_97; x_21 = x_13; x_22 = x_14; @@ -80433,8 +80433,8 @@ lean_dec_ref(x_104); x_106 = lean_ctor_get(x_105, 1); lean_inc(x_106); lean_dec(x_105); -x_18 = x_73; -x_19 = x_61; +x_18 = x_61; +x_19 = x_73; x_20 = x_106; x_21 = x_13; x_22 = x_14; @@ -81045,7 +81045,7 @@ x_27 = lean_box_usize(x_26); x_28 = lean_box_usize(x_20); x_29 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addDefaults___lam__0___boxed), 18, 10); lean_closure_set(x_29, 0, x_25); -lean_closure_set(x_29, 1, x_19); +lean_closure_set(x_29, 1, x_21); lean_closure_set(x_29, 2, x_22); lean_closure_set(x_29, 3, x_2); lean_closure_set(x_29, 4, x_3); @@ -81054,7 +81054,7 @@ lean_closure_set(x_29, 6, x_18); lean_closure_set(x_29, 7, x_17); lean_closure_set(x_29, 8, x_27); lean_closure_set(x_29, 9, x_28); -x_30 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_21, x_24, x_29, x_16, x_5, x_6, x_7, x_8, x_9, x_10); +x_30 = l_Lean_Meta_withLCtx___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCtor_spec__2___redArg(x_19, x_24, x_29, x_16, x_5, x_6, x_7, x_8, x_9, x_10); return x_30; } else @@ -81102,9 +81102,9 @@ x_42 = lean_nat_dec_lt(x_18, x_36); if (x_42 == 0) { lean_dec(x_36); -x_19 = x_40; +x_19 = x_35; x_20 = x_39; -x_21 = x_35; +x_21 = x_40; x_22 = x_41; goto block_34; } @@ -81115,9 +81115,9 @@ x_43 = lean_nat_dec_le(x_36, x_36); if (x_43 == 0) { lean_dec(x_36); -x_19 = x_40; +x_19 = x_35; x_20 = x_39; -x_21 = x_35; +x_21 = x_40; x_22 = x_41; goto block_34; } @@ -81127,9 +81127,9 @@ size_t x_44; lean_object* x_45; x_44 = lean_usize_of_nat(x_36); lean_dec(x_36); x_45 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkFlatCtorExpr_spec__3(x_17, x_39, x_44, x_41); -x_19 = x_40; +x_19 = x_35; x_20 = x_39; -x_21 = x_35; +x_21 = x_40; x_22 = x_45; goto block_34; } @@ -82023,7 +82023,7 @@ lean_inc_ref(x_6); x_13 = l_Lean_Meta_isProp(x_6, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; uint8_t x_99; lean_object* x_100; uint8_t x_101; uint8_t x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_163; uint8_t x_164; uint8_t x_165; uint8_t x_185; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t 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_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; uint8_t x_99; uint8_t x_100; uint8_t x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_163; uint8_t x_164; uint8_t x_165; uint8_t x_185; x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); lean_dec_ref(x_13); @@ -82078,12 +82078,12 @@ goto block_184; block_39: { lean_object* x_30; -lean_inc(x_22); -x_30 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCoercionToCopiedParent_spec__0(x_22, x_18, x_23, x_25, x_26, x_27, x_28); +lean_inc(x_21); +x_30 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCoercionToCopiedParent_spec__0(x_21, x_18, x_22, x_25, x_26, x_27, x_28); lean_dec(x_28); lean_dec(x_26); lean_dec_ref(x_25); -lean_dec(x_23); +lean_dec(x_22); lean_dec(x_18); if (lean_obj_tag(x_30) == 0) { @@ -82095,8 +82095,8 @@ lean_object* x_32; lean_object* x_33; x_32 = lean_ctor_get(x_30, 0); lean_dec(x_32); x_33 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_33, 0, x_21); -lean_ctor_set(x_33, 1, x_22); +lean_ctor_set(x_33, 0, x_23); +lean_ctor_set(x_33, 1, x_21); lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_24); lean_ctor_set(x_30, 0, x_33); return x_30; @@ -82106,8 +82106,8 @@ else lean_object* x_34; lean_object* x_35; lean_dec(x_30); x_34 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_34, 0, x_21); -lean_ctor_set(x_34, 1, x_22); +lean_ctor_set(x_34, 0, x_23); +lean_ctor_set(x_34, 1, x_21); lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_24); x_35 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_35, 0, x_34); @@ -82117,7 +82117,7 @@ return x_35; else { uint8_t x_36; -lean_dec(x_22); +lean_dec(x_23); lean_dec(x_21); x_36 = !lean_is_exclusive(x_30); if (x_36 == 0) @@ -82150,7 +82150,7 @@ lean_object* x_51; uint8_t x_52; x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); lean_dec_ref(x_50); -x_52 = l_Lean_BinderInfo_isInstImplicit(x_43); +x_52 = l_Lean_BinderInfo_isInstImplicit(x_42); if (x_52 == 0) { uint8_t x_53; @@ -82159,12 +82159,12 @@ lean_dec(x_51); if (x_53 == 0) { lean_object* x_54; -lean_inc(x_41); -x_54 = l_Lean_setReducibleAttribute___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCoercionToCopiedParent_spec__1(x_41, x_45, x_46, x_47, x_48); +lean_inc(x_40); +x_54 = l_Lean_setReducibleAttribute___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_mkCoercionToCopiedParent_spec__1(x_40, x_45, x_46, x_47, x_48); lean_dec_ref(x_54); x_21 = x_40; x_22 = x_41; -x_23 = x_42; +x_23 = x_43; x_24 = x_44; x_25 = x_45; x_26 = x_46; @@ -82177,7 +82177,7 @@ else { x_21 = x_40; x_22 = x_41; -x_23 = x_42; +x_23 = x_43; x_24 = x_44; x_25 = x_45; x_26 = x_46; @@ -82192,7 +82192,7 @@ else lean_dec(x_51); x_21 = x_40; x_22 = x_41; -x_23 = x_42; +x_23 = x_43; x_24 = x_44; x_25 = x_45; x_26 = x_46; @@ -82209,7 +82209,7 @@ lean_dec(x_48); lean_dec_ref(x_47); lean_dec(x_46); lean_dec_ref(x_45); -lean_dec(x_42); +lean_dec(x_43); lean_dec(x_41); lean_dec(x_40); lean_dec(x_18); @@ -82233,21 +82233,21 @@ return x_57; block_74: { lean_object* x_70; -lean_inc(x_59); -lean_inc_ref(x_60); -x_70 = l_Lean_addDecl(x_69, x_66, x_60, x_59); +lean_inc(x_65); +lean_inc_ref(x_61); +x_70 = l_Lean_addDecl(x_69, x_68, x_61, x_65); if (lean_obj_tag(x_70) == 0) { lean_dec_ref(x_70); -x_40 = x_61; +x_40 = x_59; x_41 = x_62; -x_42 = x_64; -x_43 = x_63; -x_44 = x_66; +x_42 = x_63; +x_43 = x_66; +x_44 = x_68; x_45 = x_67; -x_46 = x_65; -x_47 = x_60; -x_48 = x_59; +x_46 = x_64; +x_47 = x_61; +x_48 = x_65; x_49 = lean_box(0); goto block_58; } @@ -82255,11 +82255,11 @@ else { uint8_t x_71; lean_dec_ref(x_67); +lean_dec(x_66); lean_dec(x_65); lean_dec(x_64); lean_dec(x_62); -lean_dec(x_61); -lean_dec_ref(x_60); +lean_dec_ref(x_61); lean_dec(x_59); lean_dec(x_18); lean_dec_ref(x_6); @@ -82284,46 +82284,46 @@ return x_73; { lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; x_90 = lean_box(0); -lean_inc(x_79); +lean_inc(x_75); x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_79); +lean_ctor_set(x_91, 0, x_75); lean_ctor_set(x_91, 1, x_90); x_92 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_92, 0, x_82); -lean_ctor_set(x_92, 1, x_84); -lean_ctor_set(x_92, 2, x_78); +lean_ctor_set(x_92, 0, x_88); +lean_ctor_set(x_92, 1, x_83); +lean_ctor_set(x_92, 2, x_84); lean_ctor_set(x_92, 3, x_91); lean_ctor_set_uint8(x_92, sizeof(void*)*4, x_89); x_93 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_93, 0, x_92); -lean_inc(x_77); -lean_inc_ref(x_76); -x_94 = l_Lean_addAndCompile(x_93, x_75, x_76, x_77); +lean_inc(x_86); +lean_inc_ref(x_77); +x_94 = l_Lean_addAndCompile(x_93, x_76, x_77, x_86); if (lean_obj_tag(x_94) == 0) { lean_dec_ref(x_94); -x_40 = x_83; -x_41 = x_79; -x_42 = x_80; +x_40 = x_75; +x_41 = x_78; +x_42 = x_79; x_43 = x_81; -x_44 = x_85; -x_45 = x_88; -x_46 = x_86; -x_47 = x_76; -x_48 = x_77; +x_44 = x_82; +x_45 = x_80; +x_46 = x_87; +x_47 = x_77; +x_48 = x_86; x_49 = lean_box(0); goto block_58; } else { uint8_t x_95; -lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); -lean_dec(x_83); -lean_dec(x_80); -lean_dec(x_79); -lean_dec(x_77); -lean_dec_ref(x_76); +lean_dec(x_81); +lean_dec_ref(x_80); +lean_dec(x_78); +lean_dec_ref(x_77); +lean_dec(x_75); lean_dec(x_18); lean_dec_ref(x_6); x_95 = !lean_is_exclusive(x_94); @@ -82346,15 +82346,15 @@ return x_97; block_162: { lean_object* x_110; -x_110 = l_Lean_Meta_mkLambdaFVars(x_100, x_7, x_103, x_99, x_103, x_99, x_101, x_105, x_106, x_107, x_108); -lean_dec_ref(x_100); +x_110 = l_Lean_Meta_mkLambdaFVars(x_102, x_7, x_101, x_99, x_101, x_99, x_103, x_105, x_106, x_107, x_108); +lean_dec_ref(x_102); if (lean_obj_tag(x_110) == 0) { lean_object* x_111; lean_object* x_112; x_111 = lean_ctor_get(x_110, 0); lean_inc(x_111); lean_dec_ref(x_110); -x_112 = l_Lean_Meta_mkLambdaFVars(x_2, x_111, x_103, x_99, x_103, x_99, x_101, x_105, x_106, x_107, x_108); +x_112 = l_Lean_Meta_mkLambdaFVars(x_2, x_111, x_101, x_99, x_101, x_99, x_103, x_105, x_106, x_107, x_108); if (lean_obj_tag(x_112) == 0) { lean_object* x_113; lean_object* x_114; uint8_t x_115; @@ -82398,20 +82398,20 @@ if (x_124 == 0) { uint8_t x_126; x_126 = 1; -x_75 = x_99; -x_76 = x_107; -x_77 = x_108; -x_78 = x_125; -x_79 = x_119; -x_80 = x_117; -x_81 = x_102; -x_82 = x_122; -x_83 = x_118; -x_84 = x_116; -x_85 = x_103; -x_86 = x_106; -x_87 = lean_box(0); -x_88 = x_105; +x_75 = x_119; +x_76 = x_99; +x_77 = x_107; +x_78 = x_117; +x_79 = x_100; +x_80 = x_105; +x_81 = x_118; +x_82 = x_101; +x_83 = x_116; +x_84 = x_125; +x_85 = lean_box(0); +x_86 = x_108; +x_87 = x_106; +x_88 = x_122; x_89 = x_126; goto block_98; } @@ -82419,20 +82419,20 @@ else { uint8_t x_127; x_127 = 0; -x_75 = x_99; -x_76 = x_107; -x_77 = x_108; -x_78 = x_125; -x_79 = x_119; -x_80 = x_117; -x_81 = x_102; -x_82 = x_122; -x_83 = x_118; -x_84 = x_116; -x_85 = x_103; -x_86 = x_106; -x_87 = lean_box(0); -x_88 = x_105; +x_75 = x_119; +x_76 = x_99; +x_77 = x_107; +x_78 = x_117; +x_79 = x_100; +x_80 = x_105; +x_81 = x_118; +x_82 = x_101; +x_83 = x_116; +x_84 = x_125; +x_85 = lean_box(0); +x_86 = x_108; +x_87 = x_106; +x_88 = x_122; x_89 = x_127; goto block_98; } @@ -82456,16 +82456,16 @@ lean_ctor_set(x_131, 1, x_116); lean_ctor_set(x_131, 2, x_130); lean_ctor_set_tag(x_114, 2); lean_ctor_set(x_114, 0, x_131); -x_59 = x_108; -x_60 = x_107; -x_61 = x_118; -x_62 = x_119; -x_63 = x_102; -x_64 = x_117; -x_65 = x_106; -x_66 = x_103; +x_59 = x_119; +x_60 = lean_box(0); +x_61 = x_107; +x_62 = x_117; +x_63 = x_100; +x_64 = x_106; +x_65 = x_108; +x_66 = x_118; x_67 = x_105; -x_68 = lean_box(0); +x_68 = x_101; x_69 = x_114; goto block_74; } @@ -82484,16 +82484,16 @@ lean_ctor_set(x_134, 2, x_133); lean_ctor_set_uint8(x_134, sizeof(void*)*3, x_99); lean_ctor_set_tag(x_114, 3); lean_ctor_set(x_114, 0, x_134); -x_59 = x_108; -x_60 = x_107; -x_61 = x_118; -x_62 = x_119; -x_63 = x_102; -x_64 = x_117; -x_65 = x_106; -x_66 = x_103; +x_59 = x_119; +x_60 = lean_box(0); +x_61 = x_107; +x_62 = x_117; +x_63 = x_100; +x_64 = x_106; +x_65 = x_108; +x_66 = x_118; x_67 = x_105; -x_68 = lean_box(0); +x_68 = x_101; x_69 = x_114; goto block_74; } @@ -82535,20 +82535,20 @@ if (x_143 == 0) { uint8_t x_145; x_145 = 1; -x_75 = x_99; -x_76 = x_107; -x_77 = x_108; -x_78 = x_144; -x_79 = x_138; -x_80 = x_136; -x_81 = x_102; -x_82 = x_141; -x_83 = x_137; -x_84 = x_135; -x_85 = x_103; -x_86 = x_106; -x_87 = lean_box(0); -x_88 = x_105; +x_75 = x_138; +x_76 = x_99; +x_77 = x_107; +x_78 = x_136; +x_79 = x_100; +x_80 = x_105; +x_81 = x_137; +x_82 = x_101; +x_83 = x_135; +x_84 = x_144; +x_85 = lean_box(0); +x_86 = x_108; +x_87 = x_106; +x_88 = x_141; x_89 = x_145; goto block_98; } @@ -82556,20 +82556,20 @@ else { uint8_t x_146; x_146 = 0; -x_75 = x_99; -x_76 = x_107; -x_77 = x_108; -x_78 = x_144; -x_79 = x_138; -x_80 = x_136; -x_81 = x_102; -x_82 = x_141; -x_83 = x_137; -x_84 = x_135; -x_85 = x_103; -x_86 = x_106; -x_87 = lean_box(0); -x_88 = x_105; +x_75 = x_138; +x_76 = x_99; +x_77 = x_107; +x_78 = x_136; +x_79 = x_100; +x_80 = x_105; +x_81 = x_137; +x_82 = x_101; +x_83 = x_135; +x_84 = x_144; +x_85 = lean_box(0); +x_86 = x_108; +x_87 = x_106; +x_88 = x_141; x_89 = x_146; goto block_98; } @@ -82593,16 +82593,16 @@ lean_ctor_set(x_150, 1, x_135); lean_ctor_set(x_150, 2, x_149); x_151 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_151, 0, x_150); -x_59 = x_108; -x_60 = x_107; -x_61 = x_137; -x_62 = x_138; -x_63 = x_102; -x_64 = x_136; -x_65 = x_106; -x_66 = x_103; +x_59 = x_138; +x_60 = lean_box(0); +x_61 = x_107; +x_62 = x_136; +x_63 = x_100; +x_64 = x_106; +x_65 = x_108; +x_66 = x_137; x_67 = x_105; -x_68 = lean_box(0); +x_68 = x_101; x_69 = x_151; goto block_74; } @@ -82621,16 +82621,16 @@ lean_ctor_set(x_154, 2, x_153); lean_ctor_set_uint8(x_154, sizeof(void*)*3, x_99); x_155 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_155, 0, x_154); -x_59 = x_108; -x_60 = x_107; -x_61 = x_137; -x_62 = x_138; -x_63 = x_102; -x_64 = x_136; -x_65 = x_106; -x_66 = x_103; +x_59 = x_138; +x_60 = lean_box(0); +x_61 = x_107; +x_62 = x_136; +x_63 = x_100; +x_64 = x_106; +x_65 = x_108; +x_66 = x_137; x_67 = x_105; -x_68 = lean_box(0); +x_68 = x_101; x_69 = x_155; goto block_74; } @@ -82731,10 +82731,10 @@ x_175 = lean_ctor_get(x_174, 0); lean_inc(x_175); lean_dec_ref(x_174); x_99 = x_163; -x_100 = x_167; -x_101 = x_169; -x_102 = x_165; -x_103 = x_168; +x_100 = x_165; +x_101 = x_168; +x_102 = x_167; +x_103 = x_169; x_104 = x_175; x_105 = x_8; x_106 = x_9; @@ -82751,10 +82751,10 @@ lean_inc(x_176); lean_dec_ref(x_174); x_177 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_setSourceInstImplicit(x_176); x_99 = x_163; -x_100 = x_167; -x_101 = x_169; -x_102 = x_165; -x_103 = x_168; +x_100 = x_165; +x_101 = x_168; +x_102 = x_167; +x_103 = x_169; x_104 = x_177; x_105 = x_8; x_106 = x_9; @@ -84365,7 +84365,7 @@ 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; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_65; uint8_t x_76; lean_object* x_77; +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_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; uint8_t x_65; uint8_t x_76; lean_object* x_77; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -84435,25 +84435,25 @@ goto block_38; block_64: { uint8_t x_60; -x_60 = lean_nat_dec_lt(x_57, x_59); +x_60 = lean_nat_dec_lt(x_58, x_59); if (x_60 == 0) { lean_dec(x_59); -lean_dec_ref(x_58); -lean_dec(x_57); +lean_dec(x_58); +lean_dec_ref(x_56); lean_dec_ref(x_45); goto block_55; } else { size_t x_61; size_t x_62; uint8_t x_63; -x_61 = lean_usize_of_nat(x_57); -lean_dec(x_57); +x_61 = lean_usize_of_nat(x_58); +lean_dec(x_58); x_62 = lean_usize_of_nat(x_59); lean_dec(x_59); lean_inc(x_6); -x_63 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_47, x_6, x_56, x_58, x_61, x_62); -lean_dec_ref(x_58); +x_63 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_47, x_6, x_57, x_56, x_61, x_62); +lean_dec_ref(x_56); if (x_63 == 0) { lean_dec_ref(x_45); @@ -84498,17 +84498,17 @@ x_74 = lean_nat_dec_le(x_71, x_73); if (x_74 == 0) { lean_dec(x_71); -x_56 = x_65; -x_57 = x_70; -x_58 = x_69; +x_56 = x_69; +x_57 = x_65; +x_58 = x_70; x_59 = x_73; goto block_64; } else { -x_56 = x_65; -x_57 = x_70; -x_58 = x_69; +x_56 = x_69; +x_57 = x_65; +x_58 = x_70; x_59 = x_71; goto block_64; } @@ -84718,7 +84718,7 @@ 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_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; uint8_t x_65; uint8_t x_76; lean_object* x_77; +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_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; uint8_t x_65; uint8_t x_76; lean_object* x_77; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -84788,25 +84788,25 @@ goto block_38; block_64: { uint8_t x_60; -x_60 = lean_nat_dec_lt(x_56, x_59); +x_60 = lean_nat_dec_lt(x_58, x_59); if (x_60 == 0) { lean_dec(x_59); -lean_dec_ref(x_57); -lean_dec(x_56); +lean_dec(x_58); +lean_dec_ref(x_56); lean_dec_ref(x_45); goto block_55; } else { size_t x_61; size_t x_62; uint8_t x_63; -x_61 = lean_usize_of_nat(x_56); -lean_dec(x_56); +x_61 = lean_usize_of_nat(x_58); +lean_dec(x_58); x_62 = lean_usize_of_nat(x_59); lean_dec(x_59); lean_inc(x_6); -x_63 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_47, x_6, x_58, x_57, x_61, x_62); -lean_dec_ref(x_57); +x_63 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_47, x_6, x_57, x_56, x_61, x_62); +lean_dec_ref(x_56); if (x_63 == 0) { lean_dec_ref(x_45); @@ -84851,17 +84851,17 @@ x_74 = lean_nat_dec_le(x_71, x_73); if (x_74 == 0) { lean_dec(x_71); -x_56 = x_70; -x_57 = x_69; -x_58 = x_65; +x_56 = x_69; +x_57 = x_65; +x_58 = x_70; x_59 = x_73; goto block_64; } else { -x_56 = x_70; -x_57 = x_69; -x_58 = x_65; +x_56 = x_69; +x_57 = x_65; +x_58 = x_70; x_59 = x_71; goto block_64; } @@ -86210,21 +86210,21 @@ goto block_48; block_58: { uint8_t x_57; -x_57 = lean_nat_dec_le(x_56, x_54); +x_57 = lean_nat_dec_le(x_56, x_55); if (x_57 == 0) { -lean_dec(x_54); +lean_dec(x_55); lean_inc(x_56); -x_49 = x_55; +x_49 = x_54; x_50 = x_56; x_51 = x_56; goto block_53; } else { -x_49 = x_55; +x_49 = x_54; x_50 = x_56; -x_51 = x_54; +x_51 = x_55; goto block_53; } } @@ -86245,16 +86245,16 @@ x_67 = lean_nat_dec_le(x_1, x_66); if (x_67 == 0) { lean_inc(x_66); -x_54 = x_66; -x_55 = x_62; +x_54 = x_62; +x_55 = x_66; x_56 = x_66; goto block_58; } else { lean_inc(x_1); -x_54 = x_66; -x_55 = x_62; +x_54 = x_62; +x_55 = x_66; x_56 = x_1; goto block_58; } @@ -86428,21 +86428,21 @@ goto block_102; block_112: { uint8_t x_111; -x_111 = lean_nat_dec_le(x_110, x_108); +x_111 = lean_nat_dec_le(x_110, x_109); if (x_111 == 0) { -lean_dec(x_108); +lean_dec(x_109); lean_inc(x_110); -x_103 = x_109; +x_103 = x_108; x_104 = x_110; x_105 = x_110; goto block_107; } else { -x_103 = x_109; +x_103 = x_108; x_104 = x_110; -x_105 = x_108; +x_105 = x_109; goto block_107; } } @@ -86463,16 +86463,16 @@ x_121 = lean_nat_dec_le(x_1, x_120); if (x_121 == 0) { lean_inc(x_120); -x_108 = x_120; -x_109 = x_116; +x_108 = x_116; +x_109 = x_120; x_110 = x_120; goto block_112; } else { lean_inc(x_1); -x_108 = x_120; -x_109 = x_116; +x_108 = x_116; +x_109 = x_120; x_110 = x_1; goto block_112; } @@ -86663,21 +86663,21 @@ goto block_159; block_169: { uint8_t x_168; -x_168 = lean_nat_dec_le(x_167, x_165); +x_168 = lean_nat_dec_le(x_167, x_166); if (x_168 == 0) { -lean_dec(x_165); +lean_dec(x_166); lean_inc(x_167); -x_160 = x_166; +x_160 = x_165; x_161 = x_167; x_162 = x_167; goto block_164; } else { -x_160 = x_166; +x_160 = x_165; x_161 = x_167; -x_162 = x_165; +x_162 = x_166; goto block_164; } } @@ -86698,16 +86698,16 @@ x_178 = lean_nat_dec_le(x_1, x_177); if (x_178 == 0) { lean_inc(x_177); -x_165 = x_177; -x_166 = x_173; +x_165 = x_173; +x_166 = x_177; x_167 = x_177; goto block_169; } else { lean_inc(x_1); -x_165 = x_177; -x_166 = x_173; +x_165 = x_173; +x_166 = x_177; x_167 = x_1; goto block_169; } @@ -88068,7 +88068,7 @@ return x_38; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; uint8_t x_63; uint8_t x_74; lean_object* x_75; +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_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_63; uint8_t x_74; lean_object* x_75; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -88143,7 +88143,7 @@ if (x_58 == 0) { lean_dec(x_57); lean_dec(x_56); -lean_dec_ref(x_54); +lean_dec_ref(x_55); lean_dec_ref(x_43); goto block_53; } @@ -88155,8 +88155,8 @@ lean_dec(x_56); x_60 = lean_usize_of_nat(x_57); lean_dec(x_57); lean_inc(x_6); -x_61 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_45, x_6, x_55, x_54, x_59, x_60); -lean_dec_ref(x_54); +x_61 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_45, x_6, x_54, x_55, x_59, x_60); +lean_dec_ref(x_55); if (x_61 == 0) { lean_dec_ref(x_43); @@ -88201,16 +88201,16 @@ x_72 = lean_nat_dec_le(x_69, x_71); if (x_72 == 0) { lean_dec(x_69); -x_54 = x_67; -x_55 = x_63; +x_54 = x_63; +x_55 = x_67; x_56 = x_68; x_57 = x_71; goto block_62; } else { -x_54 = x_67; -x_55 = x_63; +x_54 = x_63; +x_55 = x_67; x_56 = x_68; x_57 = x_69; goto block_62; @@ -88411,7 +88411,7 @@ return x_38; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_63; uint8_t x_74; lean_object* x_75; +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_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; uint8_t x_63; uint8_t x_74; lean_object* x_75; lean_dec_ref(x_11); lean_inc(x_10); lean_inc(x_6); @@ -88481,25 +88481,25 @@ goto block_36; block_62: { uint8_t x_58; -x_58 = lean_nat_dec_lt(x_55, x_57); +x_58 = lean_nat_dec_lt(x_54, x_57); if (x_58 == 0) { lean_dec(x_57); -lean_dec_ref(x_56); -lean_dec(x_55); +lean_dec_ref(x_55); +lean_dec(x_54); lean_dec_ref(x_43); goto block_53; } else { size_t x_59; size_t x_60; uint8_t x_61; -x_59 = lean_usize_of_nat(x_55); -lean_dec(x_55); +x_59 = lean_usize_of_nat(x_54); +lean_dec(x_54); x_60 = lean_usize_of_nat(x_57); lean_dec(x_57); lean_inc(x_6); -x_61 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_45, x_6, x_54, x_56, x_59, x_60); -lean_dec_ref(x_56); +x_61 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Structure_0__Lean_mergeStructureResolutionOrders_selectParent___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__13_spec__18(x_45, x_6, x_56, x_55, x_59, x_60); +lean_dec_ref(x_55); if (x_61 == 0) { lean_dec_ref(x_43); @@ -88544,17 +88544,17 @@ x_72 = lean_nat_dec_le(x_69, x_71); if (x_72 == 0) { lean_dec(x_69); -x_54 = x_63; -x_55 = x_68; -x_56 = x_67; +x_54 = x_68; +x_55 = x_67; +x_56 = x_63; x_57 = x_71; goto block_62; } else { -x_54 = x_63; -x_55 = x_68; -x_56 = x_67; +x_54 = x_68; +x_55 = x_67; +x_56 = x_63; x_57 = x_69; goto block_62; } @@ -89575,7 +89575,7 @@ goto block_24; block_51: { lean_object* x_50; -x_50 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_47, x_48, x_49); +x_50 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_48, x_47, x_49); lean_dec(x_49); x_36 = x_50; goto block_46; @@ -89583,21 +89583,21 @@ goto block_46; block_56: { uint8_t x_55; -x_55 = lean_nat_dec_le(x_54, x_53); +x_55 = lean_nat_dec_le(x_54, x_52); if (x_55 == 0) { -lean_dec(x_53); +lean_dec(x_52); lean_inc(x_54); -x_47 = x_52; -x_48 = x_54; +x_47 = x_54; +x_48 = x_53; x_49 = x_54; goto block_51; } else { -x_47 = x_52; -x_48 = x_54; -x_49 = x_53; +x_47 = x_54; +x_48 = x_53; +x_49 = x_52; goto block_51; } } @@ -89618,16 +89618,16 @@ x_65 = lean_nat_dec_le(x_1, x_64); if (x_65 == 0) { lean_inc(x_64); -x_52 = x_60; -x_53 = x_64; +x_52 = x_64; +x_53 = x_60; x_54 = x_64; goto block_56; } else { lean_inc(x_1); -x_52 = x_60; -x_53 = x_64; +x_52 = x_64; +x_53 = x_60; x_54 = x_1; goto block_56; } @@ -89787,7 +89787,7 @@ goto block_24; block_105: { lean_object* x_104; -x_104 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_101, x_102, x_103); +x_104 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_102, x_101, x_103); lean_dec(x_103); x_90 = x_104; goto block_100; @@ -89795,21 +89795,21 @@ goto block_100; block_110: { uint8_t x_109; -x_109 = lean_nat_dec_le(x_108, x_107); +x_109 = lean_nat_dec_le(x_108, x_106); if (x_109 == 0) { -lean_dec(x_107); +lean_dec(x_106); lean_inc(x_108); -x_101 = x_106; -x_102 = x_108; +x_101 = x_108; +x_102 = x_107; x_103 = x_108; goto block_105; } else { -x_101 = x_106; -x_102 = x_108; -x_103 = x_107; +x_101 = x_108; +x_102 = x_107; +x_103 = x_106; goto block_105; } } @@ -89830,16 +89830,16 @@ x_119 = lean_nat_dec_le(x_1, x_118); if (x_119 == 0) { lean_inc(x_118); -x_106 = x_114; -x_107 = x_118; +x_106 = x_118; +x_107 = x_114; x_108 = x_118; goto block_110; } else { lean_inc(x_1); -x_106 = x_114; -x_107 = x_118; +x_106 = x_118; +x_107 = x_114; x_108 = x_1; goto block_110; } @@ -90016,7 +90016,7 @@ goto block_24; block_162: { lean_object* x_161; -x_161 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_158, x_159, x_160); +x_161 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_mergeStructureResolutionOrders___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_resolveFieldDefaults_spec__5_spec__22___redArg(x_159, x_158, x_160); lean_dec(x_160); x_147 = x_161; goto block_157; @@ -90024,21 +90024,21 @@ goto block_157; block_167: { uint8_t x_166; -x_166 = lean_nat_dec_le(x_165, x_164); +x_166 = lean_nat_dec_le(x_165, x_163); if (x_166 == 0) { -lean_dec(x_164); +lean_dec(x_163); lean_inc(x_165); -x_158 = x_163; -x_159 = x_165; +x_158 = x_165; +x_159 = x_164; x_160 = x_165; goto block_162; } else { -x_158 = x_163; -x_159 = x_165; -x_160 = x_164; +x_158 = x_165; +x_159 = x_164; +x_160 = x_163; goto block_162; } } @@ -90059,16 +90059,16 @@ x_176 = lean_nat_dec_le(x_1, x_175); if (x_176 == 0) { lean_inc(x_175); -x_163 = x_171; -x_164 = x_175; +x_163 = x_175; +x_164 = x_171; x_165 = x_175; goto block_167; } else { lean_inc(x_1); -x_163 = x_171; -x_164 = x_175; +x_163 = x_175; +x_164 = x_171; x_165 = x_1; goto block_167; } @@ -90958,7 +90958,7 @@ goto _start; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addParentInstances(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_34; lean_object* x_35; uint8_t x_36; +lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_34; lean_object* x_35; uint8_t x_36; x_17 = lean_st_ref_get(x_5); x_18 = lean_unsigned_to_nat(0u); x_34 = lean_array_get_size(x_1); @@ -90998,7 +90998,7 @@ goto block_33; lean_object* x_10; size_t x_11; lean_object* x_12; x_10 = lean_box(0); x_11 = lean_array_size(x_9); -x_12 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addParentInstances_spec__2(x_10, x_9, x_11, x_7, x_10, x_2, x_3, x_4, x_5); +x_12 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addParentInstances_spec__2(x_10, x_9, x_11, x_8, x_10, x_2, x_3, x_4, x_5); lean_dec_ref(x_9); if (lean_obj_tag(x_12) == 0) { @@ -91050,8 +91050,8 @@ if (x_26 == 0) { lean_dec(x_23); lean_dec_ref(x_19); -x_7 = x_21; -x_8 = lean_box(0); +x_7 = lean_box(0); +x_8 = x_21; x_9 = x_25; goto block_16; } @@ -91063,8 +91063,8 @@ if (x_27 == 0) { lean_dec(x_23); lean_dec_ref(x_19); -x_7 = x_21; -x_8 = lean_box(0); +x_7 = lean_box(0); +x_8 = x_21; x_9 = x_25; goto block_16; } @@ -91075,8 +91075,8 @@ x_28 = lean_usize_of_nat(x_24); x_29 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Elab_Structure_0__Lean_Elab_Command_Structure_addParentInstances_spec__5(x_23, x_18, x_19, x_21, x_28, x_25); lean_dec_ref(x_19); lean_dec(x_23); -x_7 = x_21; -x_8 = lean_box(0); +x_7 = lean_box(0); +x_8 = x_21; x_9 = x_29; goto block_16; } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Do/VCGen/SuggestInvariant.c b/stage0/stdlib/Lean/Elab/Tactic/Do/VCGen/SuggestInvariant.c index 830ee945844e..655b7c321522 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Do/VCGen/SuggestInvariant.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Do/VCGen/SuggestInvariant.c @@ -11517,7 +11517,7 @@ goto block_44; if (x_30 == 0) { lean_object* x_31; -lean_dec_ref(x_28); +lean_dec_ref(x_29); x_31 = l_Lean_Elab_Tactic_SavedState_restore___redArg(x_26, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_31) == 0) { @@ -11564,12 +11564,12 @@ else lean_dec(x_27); lean_dec(x_26); lean_dec_ref(x_4); -if (lean_obj_tag(x_28) == 0) +if (lean_obj_tag(x_29) == 0) { lean_object* x_37; -x_37 = lean_ctor_get(x_28, 0); +x_37 = lean_ctor_get(x_29, 0); lean_inc(x_37); -lean_dec_ref(x_28); +lean_dec_ref(x_29); x_14 = x_37; x_15 = lean_box(0); goto block_19; @@ -11584,7 +11584,7 @@ lean_dec(x_8); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_5); -return x_28; +return x_29; } } } @@ -11596,16 +11596,16 @@ if (x_42 == 0) { uint8_t x_43; x_43 = l_Lean_Exception_isRuntime(x_40); -x_28 = x_39; -x_29 = lean_box(0); +x_28 = lean_box(0); +x_29 = x_39; x_30 = x_43; goto block_38; } else { lean_dec_ref(x_40); -x_28 = x_39; -x_29 = lean_box(0); +x_28 = lean_box(0); +x_29 = x_39; x_30 = x_42; goto block_38; } diff --git a/stage0/stdlib/Lean/Elab/Tactic/RCases.c b/stage0/stdlib/Lean/Elab/Tactic/RCases.c index 58e8565c1c43..3a07bf7d33dd 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/RCases.c +++ b/stage0/stdlib/Lean/Elab/Tactic/RCases.c @@ -5043,7 +5043,7 @@ lean_inc_ref(x_6); x_20 = l_Lean_Meta_getFunInfo(x_18, x_19, x_6, x_7, x_8, x_9); 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_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_75; lean_object* x_76; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_97; +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_75; lean_object* x_76; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_97; x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); lean_dec_ref(x_20); @@ -5075,7 +5075,7 @@ goto block_100; block_68: { lean_object* x_28; uint8_t x_29; -x_28 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructor(x_27, x_22, x_24, x_2, x_25); +x_28 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructor(x_27, x_22, x_26, x_2, x_24); lean_dec_ref(x_22); x_29 = !lean_is_exclusive(x_28); if (x_29 == 0) @@ -5088,7 +5088,7 @@ x_33 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_33, 0, x_30); lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); x_34 = lean_array_push(x_3, x_33); -x_35 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructors(x_1, x_2, x_34, x_15, x_26, x_6, x_7, x_8, x_9); +x_35 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructors(x_1, x_2, x_34, x_15, x_25, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_35) == 0) { uint8_t x_36; @@ -5202,7 +5202,7 @@ x_56 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_56, 0, x_53); lean_ctor_set_uint8(x_56, sizeof(void*)*1, x_55); x_57 = lean_array_push(x_3, x_56); -x_58 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructors(x_1, x_2, x_57, x_15, x_26, x_6, x_7, x_8, x_9); +x_58 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_processConstructors(x_1, x_2, x_57, x_15, x_25, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_58) == 0) { lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; @@ -5267,9 +5267,9 @@ lean_object* x_73; x_73 = lean_ctor_get(x_69, 0); lean_inc(x_73); lean_dec_ref(x_69); -x_24 = x_70; -x_25 = x_71; -x_26 = x_72; +x_24 = x_71; +x_25 = x_72; +x_26 = x_70; x_27 = x_73; goto block_68; } @@ -16278,7 +16278,7 @@ goto block_42; block_19: { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_14 = l_Array_toSubarray___redArg(x_10, x_12, x_13); +x_14 = l_Array_toSubarray___redArg(x_8, x_12, x_13); x_15 = l_Subarray_toArray___redArg(x_14); x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_15); @@ -16325,9 +16325,9 @@ x_34 = lean_array_get_size(x_25); x_35 = lean_nat_dec_le(x_32, x_20); if (x_35 == 0) { -x_8 = lean_box(0); +x_8 = x_25; x_9 = x_26; -x_10 = x_25; +x_10 = lean_box(0); x_11 = x_33; x_12 = x_32; x_13 = x_34; @@ -16336,9 +16336,9 @@ goto block_19; else { lean_dec(x_32); -x_8 = lean_box(0); +x_8 = x_25; x_9 = x_26; -x_10 = x_25; +x_10 = lean_box(0); x_11 = x_33; x_12 = x_20; x_13 = x_34; @@ -16891,10 +16891,10 @@ lean_dec_ref(x_45); x_47 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_name_x3f(x_33); if (lean_obj_tag(x_31) == 0) { -x_12 = lean_box(0); -x_13 = x_46; -x_14 = x_47; -x_15 = x_33; +x_12 = x_33; +x_13 = x_47; +x_14 = lean_box(0); +x_15 = x_46; x_16 = x_44; goto block_23; } @@ -16909,10 +16909,10 @@ x_49 = lean_ctor_get(x_31, 0); x_50 = l_Lean_TSyntax_getId(x_49); lean_dec(x_49); lean_ctor_set(x_31, 0, x_50); -x_12 = lean_box(0); -x_13 = x_46; -x_14 = x_47; -x_15 = x_33; +x_12 = x_33; +x_13 = x_47; +x_14 = lean_box(0); +x_15 = x_46; x_16 = x_31; goto block_23; } @@ -16926,10 +16926,10 @@ x_52 = l_Lean_TSyntax_getId(x_51); lean_dec(x_51); x_53 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_53, 0, x_52); -x_12 = lean_box(0); -x_13 = x_46; -x_14 = x_47; -x_15 = x_33; +x_12 = x_33; +x_13 = x_47; +x_14 = lean_box(0); +x_15 = x_46; x_16 = x_53; goto block_23; } @@ -17008,11 +17008,11 @@ return x_59; { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_17 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_17, 0, x_13); -lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_13); lean_ctor_set(x_17, 2, x_16); x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_15); +lean_ctor_set(x_18, 0, x_12); lean_ctor_set(x_18, 1, x_17); x_19 = lean_unsigned_to_nat(1u); x_20 = lean_nat_add(x_3, x_19); @@ -18228,28 +18228,28 @@ if (x_46 == 0) lean_object* x_47; lean_dec(x_6); x_47 = lean_box(0); -x_16 = x_38; -x_17 = x_41; -x_18 = x_39; -x_19 = x_42; -x_20 = x_40; -x_21 = x_37; -x_22 = lean_box(0); -x_23 = x_44; +x_16 = x_39; +x_17 = x_42; +x_18 = x_44; +x_19 = x_40; +x_20 = lean_box(0); +x_21 = x_41; +x_22 = x_38; +x_23 = x_37; x_24 = x_36; x_25 = x_47; goto block_28; } else { -x_16 = x_38; -x_17 = x_41; -x_18 = x_39; -x_19 = x_42; -x_20 = x_40; -x_21 = x_37; -x_22 = lean_box(0); -x_23 = x_44; +x_16 = x_39; +x_17 = x_42; +x_18 = x_44; +x_19 = x_40; +x_20 = lean_box(0); +x_21 = x_41; +x_22 = x_38; +x_23 = x_37; x_24 = x_36; x_25 = x_6; goto block_28; @@ -18439,14 +18439,14 @@ return x_100; if (lean_obj_tag(x_24) == 0) { lean_object* x_26; -x_26 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_rintroContinue___redArg(x_1, x_2, x_3, x_25, x_23, x_7, x_4, x_8, x_21, x_16, x_18, x_20, x_17, x_19); +x_26 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_rintroContinue___redArg(x_1, x_2, x_3, x_25, x_18, x_7, x_4, x_8, x_23, x_22, x_16, x_19, x_21, x_17); return x_26; } else { lean_object* x_27; lean_dec(x_7); -x_27 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_rintroContinue___redArg(x_1, x_2, x_3, x_25, x_23, x_24, x_4, x_8, x_21, x_16, x_18, x_20, x_17, x_19); +x_27 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_rintroContinue___redArg(x_1, x_2, x_3, x_25, x_18, x_24, x_4, x_8, x_23, x_22, x_16, x_19, x_21, x_17); return x_27; } } @@ -19764,17 +19764,17 @@ goto block_154; block_59: { lean_object* x_47; -x_47 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_36, x_41, x_43, x_45, x_40); +x_47 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_40, x_38, x_39, x_43, x_45); if (lean_obj_tag(x_47) == 0) { lean_object* x_48; lean_object* x_49; lean_object* x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); lean_dec_ref(x_47); -x_49 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_typed_x3f(x_34, x_46, x_38); -lean_dec(x_38); -x_50 = l_Lean_Syntax_TSepArray_getElems___redArg(x_35); -lean_dec_ref(x_35); +x_49 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_typed_x3f(x_34, x_46, x_41); +lean_dec(x_41); +x_50 = l_Lean_Syntax_TSepArray_getElems___redArg(x_44); +lean_dec_ref(x_44); x_51 = lean_array_size(x_50); x_52 = 0; x_53 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalObtain_spec__0(x_51, x_52, x_50); @@ -19783,22 +19783,22 @@ x_54 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_RCases_0__Lean_El lean_closure_set(x_54, 0, x_53); lean_closure_set(x_54, 1, x_49); lean_closure_set(x_54, 2, x_48); -x_55 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalRCases_spec__2___redArg(x_48, x_54, x_42, x_36, x_37, x_39, x_41, x_43, x_45, x_40); +x_55 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalRCases_spec__2___redArg(x_48, x_54, x_36, x_40, x_35, x_37, x_38, x_39, x_43, x_45); return x_55; } else { uint8_t x_56; lean_dec_ref(x_46); -lean_dec_ref(x_45); -lean_dec(x_43); -lean_dec_ref(x_42); -lean_dec_ref(x_41); +lean_dec(x_45); +lean_dec_ref(x_44); +lean_dec_ref(x_43); +lean_dec(x_41); lean_dec(x_40); lean_dec(x_39); -lean_dec(x_38); -lean_dec_ref(x_37); -lean_dec(x_36); +lean_dec_ref(x_38); +lean_dec(x_37); +lean_dec_ref(x_36); lean_dec_ref(x_35); lean_dec(x_34); x_56 = !lean_is_exclusive(x_47); @@ -19820,29 +19820,29 @@ return x_58; } block_84: { -if (lean_obj_tag(x_61) == 1) +if (lean_obj_tag(x_68) == 1) { if (lean_obj_tag(x_70) == 0) { lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_61, 0); +x_72 = lean_ctor_get(x_68, 0); lean_inc(x_72); -lean_dec_ref(x_61); +lean_dec_ref(x_68); x_73 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_instInhabited___closed__1; lean_inc(x_34); x_74 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_74, 0, x_34); lean_ctor_set(x_74, 1, x_73); -x_35 = x_72; -x_36 = x_60; +x_35 = x_60; +x_36 = x_61; x_37 = x_62; x_38 = x_63; x_39 = x_64; x_40 = x_65; -x_41 = x_66; -x_42 = x_67; -x_43 = x_68; -x_44 = lean_box(0); +x_41 = x_67; +x_42 = lean_box(0); +x_43 = x_66; +x_44 = x_72; x_45 = x_69; x_46 = x_74; goto block_59; @@ -19850,22 +19850,22 @@ goto block_59; else { lean_object* x_75; lean_object* x_76; -x_75 = lean_ctor_get(x_61, 0); +x_75 = lean_ctor_get(x_68, 0); lean_inc(x_75); -lean_dec_ref(x_61); +lean_dec_ref(x_68); x_76 = lean_ctor_get(x_70, 0); lean_inc(x_76); lean_dec_ref(x_70); -x_35 = x_75; -x_36 = x_60; +x_35 = x_60; +x_36 = x_61; x_37 = x_62; x_38 = x_63; x_39 = x_64; x_40 = x_65; -x_41 = x_66; -x_42 = x_67; -x_43 = x_68; -x_44 = lean_box(0); +x_41 = x_67; +x_42 = lean_box(0); +x_43 = x_66; +x_44 = x_75; x_45 = x_69; x_46 = x_76; goto block_59; @@ -19873,28 +19873,28 @@ goto block_59; } else { -lean_dec(x_61); -if (lean_obj_tag(x_63) == 1) +lean_dec(x_68); +if (lean_obj_tag(x_67) == 1) { if (lean_obj_tag(x_70) == 0) { lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_63, 0); +x_77 = lean_ctor_get(x_67, 0); lean_inc(x_77); -lean_dec_ref(x_63); +lean_dec_ref(x_67); x_78 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalObtain___closed__3; x_79 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_79, 0, x_34); lean_ctor_set(x_79, 1, x_78); x_11 = x_77; x_12 = x_60; -x_13 = x_62; -x_14 = x_64; -x_15 = x_65; -x_16 = x_66; -x_17 = x_67; -x_18 = x_68; -x_19 = lean_box(0); +x_13 = x_61; +x_14 = x_62; +x_15 = x_63; +x_16 = x_64; +x_17 = x_65; +x_18 = lean_box(0); +x_19 = x_66; x_20 = x_69; x_21 = x_79; goto block_29; @@ -19903,21 +19903,21 @@ else { lean_object* x_80; lean_object* x_81; lean_dec(x_34); -x_80 = lean_ctor_get(x_63, 0); +x_80 = lean_ctor_get(x_67, 0); lean_inc(x_80); -lean_dec_ref(x_63); +lean_dec_ref(x_67); x_81 = lean_ctor_get(x_70, 0); lean_inc(x_81); lean_dec_ref(x_70); x_11 = x_80; x_12 = x_60; -x_13 = x_62; -x_14 = x_64; -x_15 = x_65; -x_16 = x_66; -x_17 = x_67; -x_18 = x_68; -x_19 = lean_box(0); +x_13 = x_61; +x_14 = x_62; +x_15 = x_63; +x_16 = x_64; +x_17 = x_65; +x_18 = lean_box(0); +x_19 = x_66; x_20 = x_69; x_21 = x_81; goto block_29; @@ -19927,38 +19927,38 @@ else { lean_object* x_82; lean_object* x_83; lean_dec(x_70); -lean_dec_ref(x_67); -lean_dec(x_64); -lean_dec(x_63); -lean_dec_ref(x_62); -lean_dec(x_60); +lean_dec(x_67); +lean_dec(x_65); +lean_dec(x_62); +lean_dec_ref(x_61); +lean_dec_ref(x_60); lean_dec(x_34); x_82 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalObtain___closed__5; -x_83 = l_Lean_throwError___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalObtain_spec__1___redArg(x_82, x_66, x_68, x_69, x_65); -lean_dec(x_65); -lean_dec_ref(x_69); -lean_dec(x_68); +x_83 = l_Lean_throwError___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalObtain_spec__1___redArg(x_82, x_63, x_64, x_66, x_69); +lean_dec(x_69); lean_dec_ref(x_66); +lean_dec(x_64); +lean_dec_ref(x_63); return x_83; } } } block_112: { -if (lean_obj_tag(x_86) == 0) +if (lean_obj_tag(x_85) == 0) { lean_object* x_97; x_97 = lean_box(0); -x_60 = x_89; -x_61 = x_87; -x_62 = x_90; -x_63 = x_85; -x_64 = x_91; -x_65 = x_95; -x_66 = x_92; -x_67 = x_88; -x_68 = x_93; -x_69 = x_94; +x_60 = x_90; +x_61 = x_88; +x_62 = x_91; +x_63 = x_92; +x_64 = x_93; +x_65 = x_89; +x_66 = x_94; +x_67 = x_86; +x_68 = x_87; +x_69 = x_95; x_70 = x_97; x_71 = lean_box(0); goto block_84; @@ -19966,11 +19966,11 @@ goto block_84; else { uint8_t x_98; -x_98 = !lean_is_exclusive(x_86); +x_98 = !lean_is_exclusive(x_85); if (x_98 == 0) { lean_object* x_99; lean_object* x_100; -x_99 = lean_ctor_get(x_86, 0); +x_99 = lean_ctor_get(x_85, 0); x_100 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_parse(x_99, x_92, x_93, x_94, x_95); if (lean_obj_tag(x_100) == 0) { @@ -19978,25 +19978,25 @@ lean_object* x_101; x_101 = lean_ctor_get(x_100, 0); lean_inc(x_101); lean_dec_ref(x_100); -lean_ctor_set(x_86, 0, x_101); -x_60 = x_89; -x_61 = x_87; -x_62 = x_90; -x_63 = x_85; -x_64 = x_91; -x_65 = x_95; -x_66 = x_92; -x_67 = x_88; -x_68 = x_93; -x_69 = x_94; -x_70 = x_86; +lean_ctor_set(x_85, 0, x_101); +x_60 = x_90; +x_61 = x_88; +x_62 = x_91; +x_63 = x_92; +x_64 = x_93; +x_65 = x_89; +x_66 = x_94; +x_67 = x_86; +x_68 = x_87; +x_69 = x_95; +x_70 = x_85; x_71 = lean_box(0); goto block_84; } else { uint8_t x_102; -lean_free_object(x_86); +lean_free_object(x_85); lean_dec(x_95); lean_dec_ref(x_94); lean_dec(x_93); @@ -20006,7 +20006,7 @@ lean_dec_ref(x_90); lean_dec(x_89); lean_dec_ref(x_88); lean_dec(x_87); -lean_dec(x_85); +lean_dec(x_86); lean_dec(x_34); x_102 = !lean_is_exclusive(x_100); if (x_102 == 0) @@ -20028,9 +20028,9 @@ return x_104; else { lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_86, 0); +x_105 = lean_ctor_get(x_85, 0); lean_inc(x_105); -lean_dec(x_86); +lean_dec(x_85); x_106 = l___private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_RCasesPatt_parse(x_105, x_92, x_93, x_94, x_95); if (lean_obj_tag(x_106) == 0) { @@ -20040,16 +20040,16 @@ lean_inc(x_107); lean_dec_ref(x_106); x_108 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_108, 0, x_107); -x_60 = x_89; -x_61 = x_87; -x_62 = x_90; -x_63 = x_85; -x_64 = x_91; -x_65 = x_95; -x_66 = x_92; -x_67 = x_88; -x_68 = x_93; -x_69 = x_94; +x_60 = x_90; +x_61 = x_88; +x_62 = x_91; +x_63 = x_92; +x_64 = x_93; +x_65 = x_89; +x_66 = x_94; +x_67 = x_86; +x_68 = x_87; +x_69 = x_95; x_70 = x_108; x_71 = lean_box(0); goto block_84; @@ -20066,7 +20066,7 @@ lean_dec_ref(x_90); lean_dec(x_89); lean_dec_ref(x_88); lean_dec(x_87); -lean_dec(x_85); +lean_dec(x_86); lean_dec(x_34); x_109 = lean_ctor_get(x_106, 0); lean_inc(x_109); @@ -20127,8 +20127,8 @@ x_132 = l_Lean_Syntax_getArgs(x_131); lean_dec(x_131); x_133 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_133, 0, x_132); -x_85 = x_116; -x_86 = x_115; +x_85 = x_115; +x_86 = x_116; x_87 = x_133; x_88 = x_117; x_89 = x_118; @@ -20147,8 +20147,8 @@ else lean_object* x_134; lean_dec(x_127); x_134 = lean_box(0); -x_85 = x_116; -x_86 = x_115; +x_85 = x_115; +x_86 = x_116; x_87 = x_134; x_88 = x_117; x_89 = x_118; @@ -20237,7 +20237,7 @@ goto block_135; block_29: { lean_object* x_22; -x_22 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_12, x_16, x_18, x_20, x_15); +x_22 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_17, x_15, x_16, x_19, x_20); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -20249,21 +20249,21 @@ x_24 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_RCases_0__Lean_El lean_closure_set(x_24, 0, x_21); lean_closure_set(x_24, 1, x_11); lean_closure_set(x_24, 2, x_23); -x_25 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalRCases_spec__2___redArg(x_23, x_24, x_17, x_12, x_13, x_14, x_16, x_18, x_20, x_15); +x_25 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_RCases_0__Lean_Elab_Tactic_RCases_evalRCases_spec__2___redArg(x_23, x_24, x_13, x_17, x_12, x_14, x_15, x_16, x_19, x_20); return x_25; } else { uint8_t x_26; lean_dec_ref(x_21); -lean_dec_ref(x_20); -lean_dec(x_18); -lean_dec_ref(x_17); -lean_dec_ref(x_16); -lean_dec(x_15); +lean_dec(x_20); +lean_dec_ref(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec_ref(x_15); lean_dec(x_14); lean_dec_ref(x_13); -lean_dec(x_12); +lean_dec_ref(x_12); lean_dec(x_11); x_26 = !lean_is_exclusive(x_22); if (x_26 == 0) diff --git a/stage0/stdlib/Lean/Elab/Tactic/Try.c b/stage0/stdlib/Lean/Elab/Tactic/Try.c index fd9f5fbf6bb4..86401059cb01 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Try.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Try.c @@ -20288,8 +20288,8 @@ return x_176; { lean_object* x_27; lean_object* x_28; x_27 = lean_box(0); -x_28 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_go(x_1, x_26, x_17, x_15, x_27, x_16, x_13, x_19, x_22, x_14, x_18, x_23, x_24, x_25, x_21); -lean_dec_ref(x_26); +x_28 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_go(x_1, x_25, x_21, x_19, x_27, x_15, x_13, x_22, x_14, x_24, x_23, x_16, x_17, x_26, x_20); +lean_dec_ref(x_25); if (lean_obj_tag(x_28) == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; @@ -20299,7 +20299,7 @@ lean_dec_ref(x_28); x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); lean_dec(x_29); -x_31 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_30, x_23, x_24, x_25, x_21); +x_31 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_30, x_16, x_17, x_26, x_20); lean_dec(x_30); return x_31; } @@ -20328,12 +20328,12 @@ return x_34; if (x_50 == 0) { lean_object* x_51; -lean_dec_ref(x_49); -lean_dec(x_40); -lean_dec(x_38); +lean_dec_ref(x_48); +lean_dec(x_44); +lean_dec(x_42); lean_dec(x_1); -x_51 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_39, x_46, x_47, x_48, x_44); -lean_dec_ref(x_39); +x_51 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_38, x_39, x_40, x_49, x_43); +lean_dec_ref(x_38); return x_51; } else @@ -20343,9 +20343,9 @@ x_14 = x_37; x_15 = x_38; x_16 = x_39; x_17 = x_40; -x_18 = x_41; +x_18 = lean_box(0); x_19 = x_42; -x_20 = lean_box(0); +x_20 = x_43; x_21 = x_44; x_22 = x_45; x_23 = x_46; @@ -20358,7 +20358,7 @@ goto block_35; block_80: { uint8_t x_73; -x_73 = l_Array_isEmpty___redArg(x_61); +x_73 = l_Array_isEmpty___redArg(x_60); if (x_73 == 0) { x_36 = x_58; @@ -20366,15 +20366,15 @@ x_37 = x_59; x_38 = x_60; x_39 = x_61; x_40 = x_62; -x_41 = x_63; +x_41 = lean_box(0); x_42 = x_64; -x_43 = lean_box(0); +x_43 = x_65; x_44 = x_66; x_45 = x_67; x_46 = x_68; x_47 = x_69; -x_48 = x_70; -x_49 = x_71; +x_48 = x_71; +x_49 = x_70; x_50 = x_73; goto block_52; } @@ -20382,16 +20382,16 @@ else { lean_object* x_74; uint8_t x_75; x_74 = lean_array_get_size(x_71); -x_75 = lean_nat_dec_lt(x_62, x_74); +x_75 = lean_nat_dec_lt(x_66, x_74); if (x_75 == 0) { lean_object* x_76; lean_dec_ref(x_71); -lean_dec(x_62); -lean_dec(x_60); +lean_dec(x_66); +lean_dec(x_64); lean_dec(x_1); -x_76 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_61, x_68, x_69, x_70, x_66); -lean_dec_ref(x_61); +x_76 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_60, x_61, x_62, x_70, x_65); +lean_dec_ref(x_60); return x_76; } else @@ -20400,11 +20400,11 @@ if (x_75 == 0) { lean_object* x_77; lean_dec_ref(x_71); -lean_dec(x_62); -lean_dec(x_60); +lean_dec(x_66); +lean_dec(x_64); lean_dec(x_1); -x_77 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_61, x_68, x_69, x_70, x_66); -lean_dec_ref(x_61); +x_77 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_60, x_61, x_62, x_70, x_65); +lean_dec_ref(x_60); return x_77; } else @@ -20417,15 +20417,15 @@ x_37 = x_59; x_38 = x_60; x_39 = x_61; x_40 = x_62; -x_41 = x_63; +x_41 = lean_box(0); x_42 = x_64; -x_43 = lean_box(0); +x_43 = x_65; x_44 = x_66; x_45 = x_67; x_46 = x_68; x_47 = x_69; -x_48 = x_70; -x_49 = x_71; +x_48 = x_71; +x_49 = x_70; x_50 = x_79; goto block_52; } @@ -20435,43 +20435,43 @@ goto block_52; block_110: { lean_object* x_95; size_t x_96; lean_object* x_97; -lean_inc_ref(x_83); -x_95 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_getKindsSolvedAll(x_83); +lean_inc_ref(x_81); +x_95 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_getKindsSolvedAll(x_81); x_96 = lean_array_size(x_95); -lean_inc(x_81); +lean_inc(x_82); lean_inc(x_1); -x_97 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_spec__7(x_1, x_83, x_81, x_95, x_96, x_57, x_84, x_85, x_86, x_87, x_88, x_89, x_90, x_91, x_92, x_93); +x_97 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_spec__7(x_1, x_81, x_82, x_95, x_96, x_57, x_84, x_85, x_86, x_87, x_88, x_89, x_90, x_91, x_92, x_93); if (lean_obj_tag(x_97) == 0) { lean_object* x_98; size_t x_99; lean_object* x_100; uint8_t x_101; x_98 = lean_ctor_get(x_97, 0); lean_inc(x_98); lean_dec_ref(x_97); -x_99 = lean_array_size(x_83); -x_100 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_spec__8(x_95, x_99, x_57, x_83); +x_99 = lean_array_size(x_81); +x_100 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkChainResult_spec__8(x_95, x_99, x_57, x_81); lean_dec_ref(x_95); x_101 = l_Array_isEmpty___redArg(x_98); if (x_101 == 0) { lean_object* x_102; uint8_t x_103; x_102 = lean_array_get_size(x_100); -x_103 = lean_nat_dec_lt(x_82, x_102); +x_103 = lean_nat_dec_lt(x_83, x_102); if (x_103 == 0) { x_13 = x_85; -x_14 = x_88; -x_15 = x_81; -x_16 = x_98; -x_17 = x_82; -x_18 = x_89; -x_19 = x_86; -x_20 = lean_box(0); -x_21 = x_93; -x_22 = x_87; -x_23 = x_90; -x_24 = x_91; -x_25 = x_92; -x_26 = x_100; +x_14 = x_87; +x_15 = x_98; +x_16 = x_90; +x_17 = x_91; +x_18 = lean_box(0); +x_19 = x_82; +x_20 = x_93; +x_21 = x_83; +x_22 = x_86; +x_23 = x_89; +x_24 = x_88; +x_25 = x_100; +x_26 = x_92; goto block_35; } else @@ -20479,19 +20479,19 @@ else if (x_103 == 0) { x_13 = x_85; -x_14 = x_88; -x_15 = x_81; -x_16 = x_98; -x_17 = x_82; -x_18 = x_89; -x_19 = x_86; -x_20 = lean_box(0); -x_21 = x_93; -x_22 = x_87; -x_23 = x_90; -x_24 = x_91; -x_25 = x_92; -x_26 = x_100; +x_14 = x_87; +x_15 = x_98; +x_16 = x_90; +x_17 = x_91; +x_18 = lean_box(0); +x_19 = x_82; +x_20 = x_93; +x_21 = x_83; +x_22 = x_86; +x_23 = x_89; +x_24 = x_88; +x_25 = x_100; +x_26 = x_92; goto block_35; } else @@ -20502,35 +20502,35 @@ x_105 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__pri if (x_105 == 0) { x_13 = x_85; -x_14 = x_88; -x_15 = x_81; -x_16 = x_98; -x_17 = x_82; -x_18 = x_89; -x_19 = x_86; -x_20 = lean_box(0); -x_21 = x_93; -x_22 = x_87; -x_23 = x_90; -x_24 = x_91; -x_25 = x_92; -x_26 = x_100; +x_14 = x_87; +x_15 = x_98; +x_16 = x_90; +x_17 = x_91; +x_18 = lean_box(0); +x_19 = x_82; +x_20 = x_93; +x_21 = x_83; +x_22 = x_86; +x_23 = x_89; +x_24 = x_88; +x_25 = x_100; +x_26 = x_92; goto block_35; } else { x_58 = x_85; -x_59 = x_88; -x_60 = x_81; -x_61 = x_98; -x_62 = x_82; -x_63 = x_89; -x_64 = x_86; -x_65 = lean_box(0); -x_66 = x_93; -x_67 = x_87; -x_68 = x_90; -x_69 = x_91; +x_59 = x_87; +x_60 = x_98; +x_61 = x_90; +x_62 = x_91; +x_63 = lean_box(0); +x_64 = x_82; +x_65 = x_93; +x_66 = x_83; +x_67 = x_86; +x_68 = x_89; +x_69 = x_88; x_70 = x_92; x_71 = x_100; x_72 = x_101; @@ -20544,17 +20544,17 @@ else uint8_t x_106; x_106 = 0; x_58 = x_85; -x_59 = x_88; -x_60 = x_81; -x_61 = x_98; -x_62 = x_82; -x_63 = x_89; -x_64 = x_86; -x_65 = lean_box(0); -x_66 = x_93; -x_67 = x_87; -x_68 = x_90; -x_69 = x_91; +x_59 = x_87; +x_60 = x_98; +x_61 = x_90; +x_62 = x_91; +x_63 = lean_box(0); +x_64 = x_82; +x_65 = x_93; +x_66 = x_83; +x_67 = x_86; +x_68 = x_89; +x_69 = x_88; x_70 = x_92; x_71 = x_100; x_72 = x_106; @@ -20565,9 +20565,9 @@ else { uint8_t x_107; lean_dec_ref(x_95); -lean_dec_ref(x_83); +lean_dec(x_83); lean_dec(x_82); -lean_dec(x_81); +lean_dec_ref(x_81); lean_dec(x_1); x_107 = !lean_is_exclusive(x_97); if (x_107 == 0) @@ -20614,9 +20614,9 @@ x_133 = lean_unbox(x_130); lean_dec(x_130); if (x_133 == 0) { -x_81 = x_131; -x_82 = x_122; -x_83 = x_132; +x_81 = x_132; +x_82 = x_131; +x_83 = x_122; x_84 = x_127; x_85 = x_112; x_86 = x_113; @@ -20646,9 +20646,9 @@ x_140 = l_Lean_addTrace___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tac if (lean_obj_tag(x_140) == 0) { lean_dec_ref(x_140); -x_81 = x_131; -x_82 = x_122; -x_83 = x_132; +x_81 = x_132; +x_82 = x_131; +x_83 = x_122; x_84 = x_127; x_85 = x_112; x_86 = x_113; @@ -21446,11 +21446,11 @@ goto block_116; block_68: { lean_object* x_37; lean_object* x_38; +lean_dec(x_26); lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); -lean_dec(x_22); lean_dec(x_21); -lean_dec(x_19); x_37 = lean_box(0); x_38 = l_Lean_Elab_Tactic_replaceMainGoal___redArg(x_37, x_29, x_32, x_33, x_34, x_35); if (lean_obj_tag(x_38) == 0) @@ -21458,9 +21458,9 @@ if (lean_obj_tag(x_38) == 0) lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; lean_dec_ref(x_38); x_39 = lean_box(0); -x_40 = lean_array_size(x_24); +x_40 = lean_array_size(x_22); x_41 = 0; -x_42 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestGrindTrace_spec__1___redArg(x_20, x_39, x_24, x_40, x_41, x_39, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35); +x_42 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestGrindTrace_spec__1___redArg(x_20, x_39, x_22, x_40, x_41, x_39, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35); lean_dec(x_31); lean_dec_ref(x_30); lean_dec(x_29); @@ -21482,9 +21482,9 @@ lean_dec(x_35); lean_dec_ref(x_34); lean_dec(x_33); lean_dec_ref(x_32); -lean_dec_ref(x_24); +lean_dec_ref(x_22); lean_dec(x_18); -lean_ctor_set(x_42, 0, x_26); +lean_ctor_set(x_42, 0, x_19); return x_42; } else @@ -21497,9 +21497,9 @@ if (x_47 == 0) { lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; x_48 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_getSuggestionOfTactic___closed__2; -x_49 = lean_array_push(x_48, x_26); -x_50 = l_Array_append___redArg(x_49, x_24); -lean_dec_ref(x_24); +x_49 = lean_array_push(x_48, x_19); +x_50 = l_Array_append___redArg(x_49, x_22); +lean_dec_ref(x_22); x_51 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_50, x_32, x_33, x_34, x_35); lean_dec(x_35); lean_dec_ref(x_34); @@ -21511,13 +21511,13 @@ return x_51; else { lean_object* x_52; -lean_dec(x_26); -x_52 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_24, x_32, x_33, x_34, x_35); +lean_dec(x_19); +x_52 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_22, x_32, x_33, x_34, x_35); lean_dec(x_35); lean_dec_ref(x_34); lean_dec(x_33); lean_dec_ref(x_32); -lean_dec_ref(x_24); +lean_dec_ref(x_22); return x_52; } } @@ -21535,10 +21535,10 @@ lean_dec(x_35); lean_dec_ref(x_34); lean_dec(x_33); lean_dec_ref(x_32); -lean_dec_ref(x_24); +lean_dec_ref(x_22); lean_dec(x_18); x_55 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_55, 0, x_26); +lean_ctor_set(x_55, 0, x_19); return x_55; } else @@ -21550,9 +21550,9 @@ if (x_56 == 0) { lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; x_57 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_getSuggestionOfTactic___closed__2; -x_58 = lean_array_push(x_57, x_26); -x_59 = l_Array_append___redArg(x_58, x_24); -lean_dec_ref(x_24); +x_58 = lean_array_push(x_57, x_19); +x_59 = l_Array_append___redArg(x_58, x_22); +lean_dec_ref(x_22); x_60 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_59, x_32, x_33, x_34, x_35); lean_dec(x_35); lean_dec_ref(x_34); @@ -21564,13 +21564,13 @@ return x_60; else { lean_object* x_61; -lean_dec(x_26); -x_61 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_24, x_32, x_33, x_34, x_35); +lean_dec(x_19); +x_61 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_22, x_32, x_33, x_34, x_35); lean_dec(x_35); lean_dec_ref(x_34); lean_dec(x_33); lean_dec_ref(x_32); -lean_dec_ref(x_24); +lean_dec_ref(x_22); return x_61; } } @@ -21583,8 +21583,8 @@ lean_dec(x_35); lean_dec_ref(x_34); lean_dec(x_33); lean_dec_ref(x_32); -lean_dec(x_26); -lean_dec_ref(x_24); +lean_dec_ref(x_22); +lean_dec(x_19); lean_dec(x_18); x_62 = !lean_is_exclusive(x_42); if (x_62 == 0) @@ -21614,9 +21614,9 @@ lean_dec(x_31); lean_dec_ref(x_30); lean_dec(x_29); lean_dec_ref(x_28); -lean_dec(x_26); -lean_dec_ref(x_24); +lean_dec_ref(x_22); lean_dec(x_20); +lean_dec(x_19); lean_dec(x_18); x_65 = !lean_is_exclusive(x_38); if (x_65 == 0) @@ -21675,14 +21675,14 @@ x_91 = lean_unbox(x_88); lean_dec(x_88); if (x_91 == 0) { -x_19 = x_90; +x_19 = x_85; x_20 = x_86; -x_21 = x_90; -x_22 = x_89; +x_21 = x_89; +x_22 = x_83; x_23 = x_89; -x_24 = x_83; +x_24 = x_90; x_25 = x_89; -x_26 = x_85; +x_26 = x_90; x_27 = x_69; x_28 = x_70; x_29 = x_71; @@ -21703,14 +21703,14 @@ x_93 = l_Lean_addTrace___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tact if (lean_obj_tag(x_93) == 0) { lean_dec_ref(x_93); -x_19 = x_90; +x_19 = x_85; x_20 = x_86; -x_21 = x_90; -x_22 = x_89; +x_21 = x_89; +x_22 = x_83; x_23 = x_89; -x_24 = x_83; +x_24 = x_90; x_25 = x_89; -x_26 = x_85; +x_26 = x_90; x_27 = x_69; x_28 = x_70; x_29 = x_71; @@ -22633,7 +22633,7 @@ lean_closure_set(x_42, 3, x_19); lean_closure_set(x_42, 4, x_40); lean_closure_set(x_42, 5, x_18); lean_closure_set(x_42, 6, x_41); -x_43 = l_Lean_Elab_Tactic_Try_withOriginalHeartbeats___redArg(x_42, x_35, x_37, x_31, x_34, x_33, x_39, x_30, x_32, x_38); +x_43 = l_Lean_Elab_Tactic_Try_withOriginalHeartbeats___redArg(x_42, x_39, x_32, x_31, x_37, x_33, x_35, x_34, x_36, x_38); return x_43; } block_62: @@ -22648,16 +22648,16 @@ if (lean_obj_tag(x_57) == 0) { lean_object* x_58; x_58 = lean_box(0); -x_30 = x_51; +x_30 = lean_box(0); x_31 = x_47; -x_32 = x_52; +x_32 = x_46; x_33 = x_49; -x_34 = x_48; -x_35 = x_45; -x_36 = lean_box(0); -x_37 = x_46; +x_34 = x_51; +x_35 = x_50; +x_36 = x_52; +x_37 = x_48; x_38 = x_53; -x_39 = x_50; +x_39 = x_45; x_40 = x_58; goto block_44; } @@ -22667,16 +22667,16 @@ uint8_t x_59; x_59 = !lean_is_exclusive(x_57); if (x_59 == 0) { -x_30 = x_51; +x_30 = lean_box(0); x_31 = x_47; -x_32 = x_52; +x_32 = x_46; x_33 = x_49; -x_34 = x_48; -x_35 = x_45; -x_36 = lean_box(0); -x_37 = x_46; +x_34 = x_51; +x_35 = x_50; +x_36 = x_52; +x_37 = x_48; x_38 = x_53; -x_39 = x_50; +x_39 = x_45; x_40 = x_57; goto block_44; } @@ -22688,16 +22688,16 @@ lean_inc(x_60); lean_dec(x_57); x_61 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_61, 0, x_60); -x_30 = x_51; +x_30 = lean_box(0); x_31 = x_47; -x_32 = x_52; +x_32 = x_46; x_33 = x_49; -x_34 = x_48; -x_35 = x_45; -x_36 = lean_box(0); -x_37 = x_46; +x_34 = x_51; +x_35 = x_50; +x_36 = x_52; +x_37 = x_48; x_38 = x_53; -x_39 = x_50; +x_39 = x_45; x_40 = x_61; goto block_44; } @@ -23110,7 +23110,7 @@ return x_7; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00__private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at___00Lean_resolveGlobalConst___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestSimpAllTrace_spec__0_spec__0_spec__1_spec__4_spec__8_spec__12_spec__16___redArg(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) { _start: { -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_50; uint8_t x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; uint8_t x_94; uint8_t x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +lean_object* x_10; uint8_t 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_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; uint8_t x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; uint8_t x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -23145,15 +23145,15 @@ lean_ctor_set(x_25, 0, x_21); lean_ctor_set(x_25, 1, x_22); x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_14); +lean_ctor_set(x_26, 1, x_12); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_12); -lean_ctor_set(x_27, 1, x_13); -lean_ctor_set(x_27, 2, x_11); -lean_ctor_set(x_27, 3, x_15); +lean_ctor_set(x_27, 0, x_10); +lean_ctor_set(x_27, 1, x_16); +lean_ctor_set(x_27, 2, x_14); +lean_ctor_set(x_27, 3, x_13); lean_ctor_set(x_27, 4, x_26); -lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_16); -lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_10); +lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_15); +lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_11); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); lean_ctor_set(x_20, 6, x_28); @@ -23190,15 +23190,15 @@ lean_ctor_set(x_41, 0, x_21); lean_ctor_set(x_41, 1, x_22); x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_14); +lean_ctor_set(x_42, 1, x_12); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_12); -lean_ctor_set(x_43, 1, x_13); -lean_ctor_set(x_43, 2, x_11); -lean_ctor_set(x_43, 3, x_15); +lean_ctor_set(x_43, 0, x_10); +lean_ctor_set(x_43, 1, x_16); +lean_ctor_set(x_43, 2, x_14); +lean_ctor_set(x_43, 3, x_13); lean_ctor_set(x_43, 4, x_42); -lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_16); -lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_10); +lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_15); +lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_11); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); x_45 = lean_alloc_ctor(0, 9, 0); @@ -23228,25 +23228,25 @@ if (x_60 == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); -lean_inc_ref(x_54); -x_62 = l_Lean_FileMap_toPosition(x_54, x_56); -lean_dec(x_56); -x_63 = l_Lean_FileMap_toPosition(x_54, x_57); +lean_inc_ref(x_53); +x_62 = l_Lean_FileMap_toPosition(x_53, x_54); +lean_dec(x_54); +x_63 = l_Lean_FileMap_toPosition(x_53, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); x_65 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00Lean_Elab_Tactic_elabTryConfig_spec__0_spec__0_spec__3___redArg___closed__1; -if (x_51 == 0) +if (x_55 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); -x_10 = x_52; -x_11 = x_64; -x_12 = x_53; -x_13 = x_62; -x_14 = x_61; -x_15 = x_65; -x_16 = x_55; +x_10 = x_51; +x_11 = x_52; +x_12 = x_61; +x_13 = x_65; +x_14 = x_64; +x_15 = x_56; +x_16 = x_62; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -23263,7 +23263,7 @@ lean_object* x_67; lean_dec_ref(x_64); lean_dec_ref(x_62); lean_dec(x_61); -lean_dec_ref(x_53); +lean_dec_ref(x_51); lean_dec_ref(x_7); x_67 = lean_box(0); lean_ctor_set(x_59, 0, x_67); @@ -23272,13 +23272,13 @@ return x_59; else { lean_free_object(x_59); -x_10 = x_52; -x_11 = x_64; -x_12 = x_53; -x_13 = x_62; -x_14 = x_61; -x_15 = x_65; -x_16 = x_55; +x_10 = x_51; +x_11 = x_52; +x_12 = x_61; +x_13 = x_65; +x_14 = x_64; +x_15 = x_56; +x_16 = x_62; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -23292,24 +23292,24 @@ lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); -lean_inc_ref(x_54); -x_69 = l_Lean_FileMap_toPosition(x_54, x_56); -lean_dec(x_56); -x_70 = l_Lean_FileMap_toPosition(x_54, x_57); +lean_inc_ref(x_53); +x_69 = l_Lean_FileMap_toPosition(x_53, x_54); +lean_dec(x_54); +x_70 = l_Lean_FileMap_toPosition(x_53, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); x_72 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00Lean_Elab_Tactic_elabTryConfig_spec__0_spec__0_spec__3___redArg___closed__1; -if (x_51 == 0) +if (x_55 == 0) { lean_dec_ref(x_50); -x_10 = x_52; -x_11 = x_71; -x_12 = x_53; -x_13 = x_69; -x_14 = x_68; -x_15 = x_72; -x_16 = x_55; +x_10 = x_51; +x_11 = x_52; +x_12 = x_68; +x_13 = x_72; +x_14 = x_71; +x_15 = x_56; +x_16 = x_69; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -23326,7 +23326,7 @@ lean_object* x_74; lean_object* x_75; lean_dec_ref(x_71); lean_dec_ref(x_69); lean_dec(x_68); -lean_dec_ref(x_53); +lean_dec_ref(x_51); lean_dec_ref(x_7); x_74 = lean_box(0); x_75 = lean_alloc_ctor(0, 1, 0); @@ -23335,13 +23335,13 @@ return x_75; } else { -x_10 = x_52; -x_11 = x_71; -x_12 = x_53; -x_13 = x_69; -x_14 = x_68; -x_15 = x_72; -x_16 = x_55; +x_10 = x_51; +x_11 = x_52; +x_12 = x_68; +x_13 = x_72; +x_14 = x_71; +x_15 = x_56; +x_16 = x_69; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -23359,12 +23359,12 @@ if (lean_obj_tag(x_85) == 0) { lean_inc(x_84); x_50 = x_77; -x_51 = x_80; -x_52 = x_79; -x_53 = x_81; -x_54 = x_82; -x_55 = x_83; -x_56 = x_84; +x_51 = x_79; +x_52 = x_81; +x_53 = x_80; +x_54 = x_84; +x_55 = x_82; +x_56 = x_83; x_57 = x_84; goto block_76; } @@ -23375,12 +23375,12 @@ x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); lean_dec_ref(x_85); x_50 = x_77; -x_51 = x_80; -x_52 = x_79; -x_53 = x_81; -x_54 = x_82; -x_55 = x_83; -x_56 = x_84; +x_51 = x_79; +x_52 = x_81; +x_53 = x_80; +x_54 = x_84; +x_55 = x_82; +x_56 = x_83; x_57 = x_86; goto block_76; } @@ -23397,9 +23397,9 @@ lean_object* x_97; x_97 = lean_unsigned_to_nat(0u); x_77 = x_88; x_78 = x_95; -x_79 = x_94; -x_80 = x_89; -x_81 = x_90; +x_79 = x_89; +x_80 = x_90; +x_81 = x_94; x_82 = x_91; x_83 = x_93; x_84 = x_97; @@ -23413,9 +23413,9 @@ lean_inc(x_98); lean_dec_ref(x_96); x_77 = x_88; x_78 = x_95; -x_79 = x_94; -x_80 = x_89; -x_81 = x_90; +x_79 = x_89; +x_80 = x_90; +x_81 = x_94; x_82 = x_91; x_83 = x_93; x_84 = x_98; @@ -23429,8 +23429,8 @@ if (x_107 == 0) x_88 = x_105; x_89 = x_101; x_90 = x_102; -x_91 = x_103; -x_92 = x_104; +x_91 = x_104; +x_92 = x_103; x_93 = x_106; x_94 = x_3; goto block_99; @@ -23440,8 +23440,8 @@ else x_88 = x_105; x_89 = x_101; x_90 = x_102; -x_91 = x_103; -x_92 = x_104; +x_91 = x_104; +x_92 = x_103; x_93 = x_106; x_94 = x_100; goto block_99; @@ -23469,10 +23469,10 @@ if (x_119 == 0) lean_inc(x_113); lean_inc_ref(x_111); lean_inc_ref(x_110); -x_101 = x_114; -x_102 = x_110; -x_103 = x_111; -x_104 = x_113; +x_101 = x_110; +x_102 = x_111; +x_103 = x_113; +x_104 = x_114; x_105 = x_117; x_106 = x_109; x_107 = x_119; @@ -23486,10 +23486,10 @@ x_121 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwEr lean_inc(x_113); lean_inc_ref(x_111); lean_inc_ref(x_110); -x_101 = x_114; -x_102 = x_110; -x_103 = x_111; -x_104 = x_113; +x_101 = x_110; +x_102 = x_111; +x_103 = x_113; +x_104 = x_114; x_105 = x_117; x_106 = x_109; x_107 = x_121; @@ -25651,22 +25651,22 @@ return x_300; block_56: { 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_34, 0); +x_42 = lean_ctor_get(x_40, 0); lean_inc_ref(x_42); -lean_dec_ref(x_34); -x_43 = l_Array_append___redArg(x_29, x_41); +lean_dec_ref(x_40); +x_43 = l_Array_append___redArg(x_27, x_41); lean_dec_ref(x_41); -lean_inc(x_35); +lean_inc(x_33); x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_35); -lean_ctor_set(x_44, 1, x_40); +lean_ctor_set(x_44, 0, x_33); +lean_ctor_set(x_44, 1, x_34); lean_ctor_set(x_44, 2, x_43); -x_45 = l_Lean_Syntax_node5(x_35, x_36, x_27, x_31, x_28, x_32, x_44); -lean_inc(x_33); -lean_inc_ref(x_39); -lean_inc(x_30); +x_45 = l_Lean_Syntax_node5(x_33, x_28, x_37, x_30, x_32, x_35, x_44); +lean_inc(x_36); lean_inc_ref(x_38); -x_46 = l_Lean_Elab_Tactic_mkSimpCallStx(x_45, x_42, x_38, x_30, x_39, x_33); +lean_inc(x_31); +lean_inc_ref(x_39); +x_46 = l_Lean_Elab_Tactic_mkSimpCallStx(x_45, x_42, x_39, x_31, x_38, x_36); lean_dec_ref(x_42); if (lean_obj_tag(x_46) == 0) { @@ -25679,11 +25679,11 @@ lean_dec_ref(x_46); x_48 = lean_mk_empty_array_with_capacity(x_4); x_49 = lean_array_push(x_48, x_5); x_50 = lean_array_push(x_49, x_47); -x_51 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_50, x_38, x_30, x_39, x_33); -lean_dec(x_33); -lean_dec_ref(x_39); -lean_dec(x_30); +x_51 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_50, x_39, x_31, x_38, x_36); +lean_dec(x_36); lean_dec_ref(x_38); +lean_dec(x_31); +lean_dec_ref(x_39); lean_dec_ref(x_50); return x_51; } @@ -25696,11 +25696,11 @@ lean_inc(x_52); lean_dec_ref(x_46); x_53 = lean_mk_empty_array_with_capacity(x_6); x_54 = lean_array_push(x_53, x_52); -x_55 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_54, x_38, x_30, x_39, x_33); -lean_dec(x_33); -lean_dec_ref(x_39); -lean_dec(x_30); +x_55 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_mkTrySuggestions___redArg(x_54, x_39, x_31, x_38, x_36); +lean_dec(x_36); lean_dec_ref(x_38); +lean_dec(x_31); +lean_dec_ref(x_39); lean_dec_ref(x_54); return x_55; } @@ -25709,8 +25709,8 @@ else { lean_dec_ref(x_39); lean_dec_ref(x_38); -lean_dec(x_33); -lean_dec(x_30); +lean_dec(x_36); +lean_dec(x_31); lean_dec(x_5); return x_46; } @@ -25718,49 +25718,49 @@ return x_46; block_82: { lean_object* x_71; lean_object* x_72; -lean_inc_ref(x_59); -x_71 = l_Array_append___redArg(x_59, x_70); +lean_inc_ref(x_57); +x_71 = l_Array_append___redArg(x_57, x_70); lean_dec_ref(x_70); -lean_inc(x_69); lean_inc(x_64); +lean_inc(x_63); x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_64); -lean_ctor_set(x_72, 1, x_69); +lean_ctor_set(x_72, 0, x_63); +lean_ctor_set(x_72, 1, x_64); lean_ctor_set(x_72, 2, x_71); if (lean_obj_tag(x_7) == 1) { 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_73 = lean_ctor_get(x_7, 0); x_74 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_grindTraceToGrind___closed__2; -lean_inc(x_64); +lean_inc(x_63); x_75 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_75, 0, x_64); +lean_ctor_set(x_75, 0, x_63); lean_ctor_set(x_75, 1, x_74); -lean_inc_ref(x_59); -x_76 = l_Array_append___redArg(x_59, x_73); -lean_inc(x_69); +lean_inc_ref(x_57); +x_76 = l_Array_append___redArg(x_57, x_73); lean_inc(x_64); +lean_inc(x_63); x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_64); -lean_ctor_set(x_77, 1, x_69); +lean_ctor_set(x_77, 0, x_63); +lean_ctor_set(x_77, 1, x_64); lean_ctor_set(x_77, 2, x_76); x_78 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_grindTraceToGrind___closed__3; -lean_inc(x_64); +lean_inc(x_63); x_79 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_79, 0, x_64); +lean_ctor_set(x_79, 0, x_63); lean_ctor_set(x_79, 1, x_78); x_80 = l_Array_mkArray3___redArg(x_75, x_77, x_79); x_27 = x_57; x_28 = x_58; -x_29 = x_59; +x_29 = lean_box(0); x_30 = x_60; x_31 = x_61; -x_32 = x_72; -x_33 = x_62; -x_34 = x_63; -x_35 = x_64; +x_32 = x_62; +x_33 = x_63; +x_34 = x_64; +x_35 = x_72; x_36 = x_65; -x_37 = lean_box(0); +x_37 = x_66; x_38 = x_67; x_39 = x_68; x_40 = x_69; @@ -25773,15 +25773,15 @@ lean_object* x_81; x_81 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_grindTraceToGrind___closed__4; x_27 = x_57; x_28 = x_58; -x_29 = x_59; +x_29 = lean_box(0); x_30 = x_60; x_31 = x_61; -x_32 = x_72; -x_33 = x_62; -x_34 = x_63; -x_35 = x_64; +x_32 = x_62; +x_33 = x_63; +x_34 = x_64; +x_35 = x_72; x_36 = x_65; -x_37 = lean_box(0); +x_37 = x_66; x_38 = x_67; x_39 = x_68; x_40 = x_69; @@ -25850,19 +25850,19 @@ x_108 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_108, 0, x_106); lean_ctor_set(x_108, 1, x_107); x_109 = l_Array_mkArray1___redArg(x_108); -x_57 = x_101; -x_58 = x_104; -x_59 = x_103; -x_60 = x_86; -x_61 = x_94; -x_62 = x_88; -x_63 = x_83; -x_64 = x_97; -x_65 = x_99; -x_66 = lean_box(0); -x_67 = x_85; -x_68 = x_87; -x_69 = x_102; +x_57 = x_103; +x_58 = x_99; +x_59 = lean_box(0); +x_60 = x_94; +x_61 = x_86; +x_62 = x_104; +x_63 = x_97; +x_64 = x_102; +x_65 = x_88; +x_66 = x_101; +x_67 = x_87; +x_68 = x_85; +x_69 = x_83; x_70 = x_109; goto block_82; } @@ -25870,19 +25870,19 @@ else { lean_object* x_110; x_110 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_grindTraceToGrind___closed__4; -x_57 = x_101; -x_58 = x_104; -x_59 = x_103; -x_60 = x_86; -x_61 = x_94; -x_62 = x_88; -x_63 = x_83; -x_64 = x_97; -x_65 = x_99; -x_66 = lean_box(0); -x_67 = x_85; -x_68 = x_87; -x_69 = x_102; +x_57 = x_103; +x_58 = x_99; +x_59 = lean_box(0); +x_60 = x_94; +x_61 = x_86; +x_62 = x_104; +x_63 = x_97; +x_64 = x_102; +x_65 = x_88; +x_66 = x_101; +x_67 = x_87; +x_68 = x_85; +x_69 = x_83; x_70 = x_110; goto block_82; } @@ -26694,7 +26694,7 @@ goto block_108; block_52: { lean_object* x_37; -x_37 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_35, x_31, x_23, x_28, x_33); +x_37 = l_Lean_Elab_Tactic_getMainGoal___redArg(x_34, x_35, x_27, x_23, x_32); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; @@ -26703,24 +26703,24 @@ lean_inc(x_38); lean_dec_ref(x_37); x_39 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_grindTraceToGrind___closed__6; x_40 = lean_box(0); -x_41 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_configHasSuggestions(x_25); -lean_dec(x_25); +x_41 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_configHasSuggestions(x_24); +lean_dec(x_24); x_42 = 1; x_43 = lean_box(x_42); x_44 = lean_box(x_41); x_45 = lean_box(x_16); x_46 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestSimpAllTrace___lam__1___boxed), 26, 16); -lean_closure_set(x_46, 0, x_29); +lean_closure_set(x_46, 0, x_26); lean_closure_set(x_46, 1, x_43); lean_closure_set(x_46, 2, x_44); -lean_closure_set(x_46, 3, x_32); +lean_closure_set(x_46, 3, x_28); lean_closure_set(x_46, 4, x_1); lean_closure_set(x_46, 5, x_21); lean_closure_set(x_46, 6, x_36); lean_closure_set(x_46, 7, x_12); lean_closure_set(x_46, 8, x_13); lean_closure_set(x_46, 9, x_14); -lean_closure_set(x_46, 10, x_30); +lean_closure_set(x_46, 10, x_22); lean_closure_set(x_46, 11, x_45); lean_closure_set(x_46, 12, x_20); lean_closure_set(x_46, 13, x_39); @@ -26729,26 +26729,26 @@ lean_closure_set(x_46, 15, x_40); x_47 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Try_withOriginalHeartbeats___boxed), 12, 2); lean_closure_set(x_47, 0, lean_box(0)); lean_closure_set(x_47, 1, x_46); -x_48 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestSimpTrace_spec__0___redArg(x_38, x_47, x_27, x_34, x_35, x_22, x_24, x_31, x_23, x_28, x_33); +x_48 = l_Lean_MVarId_withContext___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestSimpTrace_spec__0___redArg(x_38, x_47, x_30, x_25, x_34, x_29, x_33, x_35, x_27, x_23, x_32); return x_48; } else { uint8_t x_49; lean_dec(x_36); -lean_dec(x_35); -lean_dec_ref(x_34); +lean_dec_ref(x_35); +lean_dec(x_34); lean_dec(x_33); lean_dec(x_32); -lean_dec_ref(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec_ref(x_28); -lean_dec_ref(x_27); -lean_dec(x_25); +lean_dec_ref(x_30); +lean_dec_ref(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec_ref(x_25); lean_dec(x_24); -lean_dec(x_23); -lean_dec_ref(x_22); +lean_dec_ref(x_23); +lean_dec(x_22); lean_dec_ref(x_19); lean_dec(x_1); x_49 = !lean_is_exclusive(x_37); @@ -26772,8 +26772,8 @@ return x_51; { lean_object* x_68; lean_object* x_69; uint8_t x_70; x_68 = lean_unsigned_to_nat(3u); -x_69 = l_Lean_Syntax_getArg(x_56, x_68); -lean_dec(x_56); +x_69 = l_Lean_Syntax_getArg(x_55, x_68); +lean_dec(x_55); x_70 = l_Lean_Syntax_isNone(x_69); if (x_70 == 0) { @@ -26794,7 +26794,7 @@ lean_dec(x_60); lean_dec_ref(x_59); lean_dec_ref(x_58); lean_dec(x_57); -lean_dec(x_55); +lean_dec(x_56); lean_dec(x_54); lean_dec(x_53); lean_dec_ref(x_19); @@ -26824,7 +26824,7 @@ lean_dec(x_60); lean_dec_ref(x_59); lean_dec_ref(x_58); lean_dec(x_57); -lean_dec(x_55); +lean_dec(x_56); lean_dec(x_54); lean_dec(x_53); lean_dec_ref(x_19); @@ -26841,20 +26841,20 @@ x_78 = l_Lean_Syntax_getArgs(x_77); lean_dec(x_77); x_79 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_79, 0, x_78); -x_22 = x_61; -x_23 = x_64; -x_24 = x_62; -x_25 = x_55; -x_26 = lean_box(0); -x_27 = x_58; -x_28 = x_65; -x_29 = x_53; -x_30 = x_57; -x_31 = x_63; -x_32 = x_54; -x_33 = x_66; -x_34 = x_59; -x_35 = x_60; +x_22 = x_57; +x_23 = x_65; +x_24 = x_56; +x_25 = x_59; +x_26 = x_53; +x_27 = x_64; +x_28 = x_54; +x_29 = x_61; +x_30 = x_58; +x_31 = lean_box(0); +x_32 = x_66; +x_33 = x_62; +x_34 = x_60; +x_35 = x_63; x_36 = x_79; goto block_52; } @@ -26865,20 +26865,20 @@ else lean_object* x_80; lean_dec(x_69); x_80 = lean_box(0); -x_22 = x_61; -x_23 = x_64; -x_24 = x_62; -x_25 = x_55; -x_26 = lean_box(0); -x_27 = x_58; -x_28 = x_65; -x_29 = x_53; -x_30 = x_57; -x_31 = x_63; -x_32 = x_54; -x_33 = x_66; -x_34 = x_59; -x_35 = x_60; +x_22 = x_57; +x_23 = x_65; +x_24 = x_56; +x_25 = x_59; +x_26 = x_53; +x_27 = x_64; +x_28 = x_54; +x_29 = x_61; +x_30 = x_58; +x_31 = lean_box(0); +x_32 = x_66; +x_33 = x_62; +x_34 = x_60; +x_35 = x_63; x_36 = x_80; goto block_52; } @@ -26975,8 +26975,8 @@ lean_ctor_set(x_106, 0, x_105); lean_inc(x_97); x_53 = x_97; x_54 = x_92; -x_55 = x_97; -x_56 = x_93; +x_55 = x_93; +x_56 = x_97; x_57 = x_106; x_58 = x_82; x_59 = x_83; @@ -26999,8 +26999,8 @@ x_107 = lean_box(0); lean_inc(x_97); x_53 = x_97; x_54 = x_92; -x_55 = x_97; -x_56 = x_93; +x_55 = x_93; +x_56 = x_97; x_57 = x_107; x_58 = x_82; x_59 = x_83; @@ -28284,17 +28284,17 @@ goto block_72; { lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_dec(x_24); +lean_dec_ref(x_23); +lean_dec(x_22); lean_dec_ref(x_20); -lean_dec(x_18); -lean_dec_ref(x_17); -lean_dec(x_16); -lean_dec_ref(x_14); +lean_dec_ref(x_16); +lean_dec(x_15); lean_dec_ref(x_13); x_25 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_evalSuggestChain___lam__0___closed__1; -x_26 = l_Lean_throwError___at___00Lean_Elab_Tactic_Try_withOriginalHeartbeats_spec__1___redArg(x_25, x_21, x_22, x_15, x_19); +x_26 = l_Lean_throwError___at___00Lean_Elab_Tactic_Try_withOriginalHeartbeats_spec__1___redArg(x_25, x_21, x_19, x_17, x_18); +lean_dec(x_18); +lean_dec_ref(x_17); lean_dec(x_19); -lean_dec_ref(x_15); -lean_dec(x_22); lean_dec_ref(x_21); x_27 = !lean_is_exclusive(x_26); if (x_27 == 0) @@ -28375,17 +28375,17 @@ x_58 = lean_nat_dec_lt(x_52, x_57); if (x_58 == 0) { x_13 = x_37; -x_14 = x_35; -x_15 = x_41; -x_16 = x_36; -x_17 = x_56; -x_18 = x_38; -x_19 = x_42; -x_20 = x_31; +x_14 = lean_box(0); +x_15 = x_47; +x_16 = x_31; +x_17 = x_41; +x_18 = x_42; +x_19 = x_40; +x_20 = x_35; x_21 = x_39; -x_22 = x_40; -x_23 = lean_box(0); -x_24 = x_47; +x_22 = x_38; +x_23 = x_56; +x_24 = x_36; goto block_30; } else @@ -28393,17 +28393,17 @@ else if (x_58 == 0) { x_13 = x_37; -x_14 = x_35; -x_15 = x_41; -x_16 = x_36; -x_17 = x_56; -x_18 = x_38; -x_19 = x_42; -x_20 = x_31; +x_14 = lean_box(0); +x_15 = x_47; +x_16 = x_31; +x_17 = x_41; +x_18 = x_42; +x_19 = x_40; +x_20 = x_35; x_21 = x_39; -x_22 = x_40; -x_23 = lean_box(0); -x_24 = x_47; +x_22 = x_38; +x_23 = x_56; +x_24 = x_36; goto block_30; } else @@ -28415,17 +28415,17 @@ x_61 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__priv if (x_61 == 0) { x_13 = x_37; -x_14 = x_35; -x_15 = x_41; -x_16 = x_36; -x_17 = x_56; -x_18 = x_38; -x_19 = x_42; -x_20 = x_31; +x_14 = lean_box(0); +x_15 = x_47; +x_16 = x_31; +x_17 = x_41; +x_18 = x_42; +x_19 = x_40; +x_20 = x_35; x_21 = x_39; -x_22 = x_40; -x_23 = lean_box(0); -x_24 = x_47; +x_22 = x_38; +x_23 = x_56; +x_24 = x_36; goto block_30; } else @@ -30043,18 +30043,18 @@ return x_75; { lean_object* x_45; x_45 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_appendSuggestion(x_4, x_31); -x_2 = x_41; +x_2 = x_43; x_3 = x_44; x_4 = x_45; -x_5 = x_40; -x_6 = x_39; -x_7 = x_35; -x_8 = x_38; -x_9 = x_37; -x_10 = x_36; -x_11 = x_43; -x_12 = x_34; -x_13 = x_42; +x_5 = x_41; +x_6 = x_34; +x_7 = x_37; +x_8 = x_33; +x_9 = x_39; +x_10 = x_40; +x_11 = x_42; +x_12 = x_35; +x_13 = x_38; goto _start; } block_61: @@ -30068,34 +30068,34 @@ if (lean_obj_tag(x_3) == 0) lean_object* x_60; x_60 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_60, 0, x_32); -x_33 = lean_box(0); -x_34 = x_55; -x_35 = x_50; -x_36 = x_53; -x_37 = x_52; -x_38 = x_51; -x_39 = x_49; -x_40 = x_48; -x_41 = x_59; -x_42 = x_56; -x_43 = x_54; +x_33 = x_51; +x_34 = x_49; +x_35 = x_55; +x_36 = lean_box(0); +x_37 = x_50; +x_38 = x_56; +x_39 = x_52; +x_40 = x_53; +x_41 = x_48; +x_42 = x_54; +x_43 = x_59; x_44 = x_60; goto block_47; } else { lean_dec(x_32); -x_33 = lean_box(0); -x_34 = x_55; -x_35 = x_50; -x_36 = x_53; -x_37 = x_52; -x_38 = x_51; -x_39 = x_49; -x_40 = x_48; -x_41 = x_59; -x_42 = x_56; -x_43 = x_54; +x_33 = x_51; +x_34 = x_49; +x_35 = x_55; +x_36 = lean_box(0); +x_37 = x_50; +x_38 = x_56; +x_39 = x_52; +x_40 = x_53; +x_41 = x_48; +x_42 = x_54; +x_43 = x_59; x_44 = x_3; goto block_47; } @@ -30233,18 +30233,18 @@ return x_121; { lean_object* x_90; x_90 = l___private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_appendSuggestion(x_4, x_76); -x_2 = x_86; +x_2 = x_88; x_3 = x_89; x_4 = x_90; -x_5 = x_85; -x_6 = x_84; -x_7 = x_80; -x_8 = x_83; -x_9 = x_82; -x_10 = x_81; -x_11 = x_88; -x_12 = x_79; -x_13 = x_87; +x_5 = x_86; +x_6 = x_79; +x_7 = x_82; +x_8 = x_78; +x_9 = x_84; +x_10 = x_85; +x_11 = x_87; +x_12 = x_80; +x_13 = x_83; goto _start; } block_106: @@ -30258,34 +30258,34 @@ if (lean_obj_tag(x_3) == 0) lean_object* x_105; x_105 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_105, 0, x_77); -x_78 = lean_box(0); -x_79 = x_100; -x_80 = x_95; -x_81 = x_98; -x_82 = x_97; -x_83 = x_96; -x_84 = x_94; -x_85 = x_93; -x_86 = x_104; -x_87 = x_101; -x_88 = x_99; +x_78 = x_96; +x_79 = x_94; +x_80 = x_100; +x_81 = lean_box(0); +x_82 = x_95; +x_83 = x_101; +x_84 = x_97; +x_85 = x_98; +x_86 = x_93; +x_87 = x_99; +x_88 = x_104; x_89 = x_105; goto block_92; } else { lean_dec(x_77); -x_78 = lean_box(0); -x_79 = x_100; -x_80 = x_95; -x_81 = x_98; -x_82 = x_97; -x_83 = x_96; -x_84 = x_94; -x_85 = x_93; -x_86 = x_104; -x_87 = x_101; -x_88 = x_99; +x_78 = x_96; +x_79 = x_94; +x_80 = x_100; +x_81 = lean_box(0); +x_82 = x_95; +x_83 = x_101; +x_84 = x_97; +x_85 = x_98; +x_86 = x_93; +x_87 = x_99; +x_88 = x_104; x_89 = x_3; goto block_92; } @@ -35231,7 +35231,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logWarning___at___00Lean_checkPrivateInPublic___at___00Lean_resolveGlobalName___at___00Lean_unresolveNameGlobal___at___00Lean_unresolveNameGlobalAvoidingLocals___at___00__private_Lean_Elab_Tactic_Try_0__Lean_Elab_Tactic_Try_toIdent_spec__0_spec__1_spec__9_spec__15_spec__19_spec__20_spec__21(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) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t 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_50; lean_object* x_51; uint8_t x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +uint8_t 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_50; uint8_t x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; uint8_t x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -35268,13 +35268,13 @@ x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_13); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_12); -lean_ctor_set(x_27, 1, x_10); -lean_ctor_set(x_27, 2, x_16); -lean_ctor_set(x_27, 3, x_11); +lean_ctor_set(x_27, 0, x_11); +lean_ctor_set(x_27, 1, x_16); +lean_ctor_set(x_27, 2, x_12); +lean_ctor_set(x_27, 3, x_14); lean_ctor_set(x_27, 4, x_26); lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_15); -lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_14); +lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_10); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); lean_ctor_set(x_20, 6, x_28); @@ -35313,13 +35313,13 @@ x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); lean_ctor_set(x_42, 1, x_13); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_12); -lean_ctor_set(x_43, 1, x_10); -lean_ctor_set(x_43, 2, x_16); -lean_ctor_set(x_43, 3, x_11); +lean_ctor_set(x_43, 0, x_11); +lean_ctor_set(x_43, 1, x_16); +lean_ctor_set(x_43, 2, x_12); +lean_ctor_set(x_43, 3, x_14); lean_ctor_set(x_43, 4, x_42); lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_15); -lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_14); +lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_10); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); x_45 = lean_alloc_ctor(0, 9, 0); @@ -35349,25 +35349,25 @@ if (x_60 == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); -lean_inc_ref(x_55); -x_62 = l_Lean_FileMap_toPosition(x_55, x_56); -lean_dec(x_56); -x_63 = l_Lean_FileMap_toPosition(x_55, x_57); +lean_inc_ref(x_56); +x_62 = l_Lean_FileMap_toPosition(x_56, x_55); +lean_dec(x_55); +x_63 = l_Lean_FileMap_toPosition(x_56, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); x_65 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00Lean_Elab_Tactic_elabTryConfig_spec__0_spec__0_spec__3___redArg___closed__1; -if (x_52 == 0) +if (x_53 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); -x_10 = x_62; -x_11 = x_65; -x_12 = x_51; +x_10 = x_51; +x_11 = x_52; +x_12 = x_64; x_13 = x_61; -x_14 = x_54; -x_15 = x_53; -x_16 = x_64; +x_14 = x_65; +x_15 = x_54; +x_16 = x_62; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -35384,7 +35384,7 @@ lean_object* x_67; lean_dec_ref(x_64); lean_dec_ref(x_62); lean_dec(x_61); -lean_dec_ref(x_51); +lean_dec_ref(x_52); lean_dec_ref(x_7); x_67 = lean_box(0); lean_ctor_set(x_59, 0, x_67); @@ -35393,13 +35393,13 @@ return x_59; else { lean_free_object(x_59); -x_10 = x_62; -x_11 = x_65; -x_12 = x_51; +x_10 = x_51; +x_11 = x_52; +x_12 = x_64; x_13 = x_61; -x_14 = x_54; -x_15 = x_53; -x_16 = x_64; +x_14 = x_65; +x_15 = x_54; +x_16 = x_62; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -35413,24 +35413,24 @@ lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); -lean_inc_ref(x_55); -x_69 = l_Lean_FileMap_toPosition(x_55, x_56); -lean_dec(x_56); -x_70 = l_Lean_FileMap_toPosition(x_55, x_57); +lean_inc_ref(x_56); +x_69 = l_Lean_FileMap_toPosition(x_56, x_55); +lean_dec(x_55); +x_70 = l_Lean_FileMap_toPosition(x_56, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); x_72 = l_Lean_addTrace___at___00__private_Lean_ExtraModUses_0__Lean_recordExtraModUseCore___at___00Lean_recordExtraModUseFromDecl___at___00Lean_Elab_Tactic_elabTryConfig_spec__0_spec__0_spec__3___redArg___closed__1; -if (x_52 == 0) +if (x_53 == 0) { lean_dec_ref(x_50); -x_10 = x_69; -x_11 = x_72; -x_12 = x_51; +x_10 = x_51; +x_11 = x_52; +x_12 = x_71; x_13 = x_68; -x_14 = x_54; -x_15 = x_53; -x_16 = x_71; +x_14 = x_72; +x_15 = x_54; +x_16 = x_69; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -35447,7 +35447,7 @@ lean_object* x_74; lean_object* x_75; lean_dec_ref(x_71); lean_dec_ref(x_69); lean_dec(x_68); -lean_dec_ref(x_51); +lean_dec_ref(x_52); lean_dec_ref(x_7); x_74 = lean_box(0); x_75 = lean_alloc_ctor(0, 1, 0); @@ -35456,13 +35456,13 @@ return x_75; } else { -x_10 = x_69; -x_11 = x_72; -x_12 = x_51; +x_10 = x_51; +x_11 = x_52; +x_12 = x_71; x_13 = x_68; -x_14 = x_54; -x_15 = x_53; -x_16 = x_71; +x_14 = x_72; +x_15 = x_54; +x_16 = x_69; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -35474,18 +35474,18 @@ goto block_49; block_87: { lean_object* x_85; -x_85 = l_Lean_Syntax_getTailPos_x3f(x_83, x_80); -lean_dec(x_83); +x_85 = l_Lean_Syntax_getTailPos_x3f(x_80, x_81); +lean_dec(x_80); if (lean_obj_tag(x_85) == 0) { lean_inc(x_84); x_50 = x_77; x_51 = x_78; -x_52 = x_81; -x_53 = x_80; -x_54 = x_79; -x_55 = x_82; -x_56 = x_84; +x_52 = x_79; +x_53 = x_82; +x_54 = x_81; +x_55 = x_84; +x_56 = x_83; x_57 = x_84; goto block_76; } @@ -35497,11 +35497,11 @@ lean_inc(x_86); lean_dec_ref(x_85); x_50 = x_77; x_51 = x_78; -x_52 = x_81; -x_53 = x_80; -x_54 = x_79; -x_55 = x_82; -x_56 = x_84; +x_52 = x_79; +x_53 = x_82; +x_54 = x_81; +x_55 = x_84; +x_56 = x_83; x_57 = x_86; goto block_76; } @@ -35509,20 +35509,20 @@ goto block_76; block_99: { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_replaceRef(x_1, x_90); -lean_dec(x_90); -x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_92); +x_95 = l_Lean_replaceRef(x_1, x_93); +lean_dec(x_93); +x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_91); if (lean_obj_tag(x_96) == 0) { lean_object* x_97; x_97 = lean_unsigned_to_nat(0u); x_77 = x_88; -x_78 = x_89; -x_79 = x_94; -x_80 = x_92; +x_78 = x_94; +x_79 = x_89; +x_80 = x_95; x_81 = x_91; -x_82 = x_93; -x_83 = x_95; +x_82 = x_90; +x_83 = x_92; x_84 = x_97; goto block_87; } @@ -35533,12 +35533,12 @@ x_98 = lean_ctor_get(x_96, 0); lean_inc(x_98); lean_dec_ref(x_96); x_77 = x_88; -x_78 = x_89; -x_79 = x_94; -x_80 = x_92; +x_78 = x_94; +x_79 = x_89; +x_80 = x_95; x_81 = x_91; -x_82 = x_93; -x_83 = x_95; +x_82 = x_90; +x_83 = x_92; x_84 = x_98; goto block_87; } @@ -35547,23 +35547,23 @@ goto block_87; { if (x_107 == 0) { -x_88 = x_105; -x_89 = x_101; -x_90 = x_102; -x_91 = x_103; -x_92 = x_106; -x_93 = x_104; +x_88 = x_101; +x_89 = x_102; +x_90 = x_103; +x_91 = x_106; +x_92 = x_104; +x_93 = x_105; x_94 = x_3; goto block_99; } else { -x_88 = x_105; -x_89 = x_101; -x_90 = x_102; -x_91 = x_103; -x_92 = x_106; -x_93 = x_104; +x_88 = x_101; +x_89 = x_102; +x_90 = x_103; +x_91 = x_106; +x_92 = x_104; +x_93 = x_105; x_94 = x_100; goto block_99; } @@ -35587,14 +35587,14 @@ x_118 = 1; x_119 = l_Lean_instBEqMessageSeverity_beq(x_3, x_118); if (x_119 == 0) { -lean_inc_ref(x_111); lean_inc(x_113); +lean_inc_ref(x_111); lean_inc_ref(x_110); -x_101 = x_110; -x_102 = x_113; +x_101 = x_117; +x_102 = x_110; x_103 = x_114; x_104 = x_111; -x_105 = x_117; +x_105 = x_113; x_106 = x_109; x_107 = x_119; goto block_108; @@ -35604,14 +35604,14 @@ else lean_object* x_120; uint8_t x_121; x_120 = l_Lean_logAt___at___00Lean_log___at___00Lean_logWarning___at___00Lean_Elab_Tactic_Try_elabRegisterTryTactic_spec__1_spec__1_spec__2___closed__0; x_121 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Elab_Tactic_elabTryConfig_spec__1_spec__5_spec__10(x_112, x_120); -lean_inc_ref(x_111); lean_inc(x_113); +lean_inc_ref(x_111); lean_inc_ref(x_110); -x_101 = x_110; -x_102 = x_113; +x_101 = x_117; +x_102 = x_110; x_103 = x_114; x_104 = x_111; -x_105 = x_117; +x_105 = x_113; x_106 = x_109; x_107 = x_121; goto block_108; diff --git a/stage0/stdlib/Lean/Elab/Term/TermElabM.c b/stage0/stdlib/Lean/Elab/Term/TermElabM.c index 37c7adc5b50e..32cfcb5efc16 100644 --- a/stage0/stdlib/Lean/Elab/Term/TermElabM.c +++ b/stage0/stdlib/Lean/Elab/Term/TermElabM.c @@ -6866,19 +6866,19 @@ goto block_102; block_77: { uint8_t x_19; -x_19 = !lean_is_exclusive(x_14); +x_19 = !lean_is_exclusive(x_13); if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_14, 6); +x_20 = lean_ctor_get(x_13, 6); lean_dec(x_20); -lean_ctor_set(x_14, 6, x_2); -lean_inc(x_11); +lean_ctor_set(x_13, 6, x_2); +lean_inc(x_16); x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withRestoreOrSaveFull___redArg___lam__0___boxed), 8, 3); lean_closure_set(x_21, 0, x_3); -lean_closure_set(x_21, 1, x_14); -lean_closure_set(x_21, 2, x_11); -x_22 = l_Lean_Meta_withRestoreOrSaveFull___redArg(x_18, x_21, x_17, x_12, x_15, x_16); +lean_closure_set(x_21, 1, x_13); +lean_closure_set(x_21, 2, x_16); +x_22 = l_Lean_Meta_withRestoreOrSaveFull___redArg(x_18, x_21, x_15, x_14, x_11, x_17); if (lean_obj_tag(x_22) == 0) { uint8_t x_23; @@ -6892,8 +6892,8 @@ if (x_25 == 0) { lean_object* x_26; lean_object* x_27; lean_object* x_28; x_26 = lean_ctor_get(x_24, 1); -x_27 = lean_st_ref_get(x_11); -lean_dec(x_11); +x_27 = lean_st_ref_get(x_16); +lean_dec(x_16); x_28 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_28, 0, x_26); lean_ctor_set(x_28, 1, x_27); @@ -6908,8 +6908,8 @@ x_30 = lean_ctor_get(x_24, 1); lean_inc(x_30); lean_inc(x_29); lean_dec(x_24); -x_31 = lean_st_ref_get(x_11); -lean_dec(x_11); +x_31 = lean_st_ref_get(x_16); +lean_dec(x_16); x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); @@ -6938,8 +6938,8 @@ if (lean_is_exclusive(x_34)) { lean_dec_ref(x_34); x_37 = lean_box(0); } -x_38 = lean_st_ref_get(x_11); -lean_dec(x_11); +x_38 = lean_st_ref_get(x_16); +lean_dec(x_16); x_39 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_39, 0, x_36); lean_ctor_set(x_39, 1, x_38); @@ -6958,7 +6958,7 @@ return x_41; else { uint8_t x_42; -lean_dec(x_11); +lean_dec(x_16); x_42 = !lean_is_exclusive(x_22); if (x_42 == 0) { @@ -6979,23 +6979,23 @@ return x_44; else { lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; uint8_t x_55; uint8_t x_56; uint8_t x_57; uint8_t x_58; uint8_t x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_45 = lean_ctor_get(x_14, 0); -x_46 = lean_ctor_get(x_14, 1); -x_47 = lean_ctor_get_uint8(x_14, sizeof(void*)*8); -x_48 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 1); -x_49 = lean_ctor_get(x_14, 2); -x_50 = lean_ctor_get(x_14, 3); -x_51 = lean_ctor_get(x_14, 4); -x_52 = lean_ctor_get(x_14, 5); -x_53 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 2); -x_54 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 3); -x_55 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 4); -x_56 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 5); -x_57 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 6); -x_58 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 7); -x_59 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 8); -x_60 = lean_ctor_get_uint8(x_14, sizeof(void*)*8 + 9); -x_61 = lean_ctor_get(x_14, 7); +x_45 = lean_ctor_get(x_13, 0); +x_46 = lean_ctor_get(x_13, 1); +x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*8); +x_48 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 1); +x_49 = lean_ctor_get(x_13, 2); +x_50 = lean_ctor_get(x_13, 3); +x_51 = lean_ctor_get(x_13, 4); +x_52 = lean_ctor_get(x_13, 5); +x_53 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 2); +x_54 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 3); +x_55 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 4); +x_56 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 5); +x_57 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 6); +x_58 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 7); +x_59 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 8); +x_60 = lean_ctor_get_uint8(x_13, sizeof(void*)*8 + 9); +x_61 = lean_ctor_get(x_13, 7); lean_inc(x_61); lean_inc(x_52); lean_inc(x_51); @@ -7003,7 +7003,7 @@ lean_inc(x_50); lean_inc(x_49); lean_inc(x_46); lean_inc(x_45); -lean_dec(x_14); +lean_dec(x_13); x_62 = lean_alloc_ctor(0, 8, 10); lean_ctor_set(x_62, 0, x_45); lean_ctor_set(x_62, 1, x_46); @@ -7023,12 +7023,12 @@ lean_ctor_set_uint8(x_62, sizeof(void*)*8 + 6, x_57); lean_ctor_set_uint8(x_62, sizeof(void*)*8 + 7, x_58); lean_ctor_set_uint8(x_62, sizeof(void*)*8 + 8, x_59); lean_ctor_set_uint8(x_62, sizeof(void*)*8 + 9, x_60); -lean_inc(x_11); +lean_inc(x_16); x_63 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withRestoreOrSaveFull___redArg___lam__0___boxed), 8, 3); lean_closure_set(x_63, 0, x_3); lean_closure_set(x_63, 1, x_62); -lean_closure_set(x_63, 2, x_11); -x_64 = l_Lean_Meta_withRestoreOrSaveFull___redArg(x_18, x_63, x_17, x_12, x_15, x_16); +lean_closure_set(x_63, 2, x_16); +x_64 = l_Lean_Meta_withRestoreOrSaveFull___redArg(x_18, x_63, x_15, x_14, x_11, x_17); 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; lean_object* x_71; lean_object* x_72; lean_object* x_73; @@ -7053,8 +7053,8 @@ if (lean_is_exclusive(x_65)) { lean_dec_ref(x_65); x_69 = lean_box(0); } -x_70 = lean_st_ref_get(x_11); -lean_dec(x_11); +x_70 = lean_st_ref_get(x_16); +lean_dec(x_16); x_71 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_71, 0, x_68); lean_ctor_set(x_71, 1, x_70); @@ -7076,7 +7076,7 @@ return x_73; else { lean_object* x_74; lean_object* x_75; lean_object* x_76; -lean_dec(x_11); +lean_dec(x_16); x_74 = lean_ctor_get(x_64, 0); lean_inc(x_74); if (lean_is_exclusive(x_64)) { @@ -7102,13 +7102,13 @@ if (lean_obj_tag(x_1) == 0) { lean_object* x_85; x_85 = lean_box(0); -x_11 = x_79; -x_12 = x_81; -x_13 = lean_box(0); -x_14 = x_78; -x_15 = x_82; -x_16 = x_83; -x_17 = x_80; +x_11 = x_82; +x_12 = lean_box(0); +x_13 = x_78; +x_14 = x_81; +x_15 = x_80; +x_16 = x_79; +x_17 = x_83; x_18 = x_85; goto block_77; } @@ -7129,13 +7129,13 @@ x_90 = lean_ctor_get(x_89, 0); lean_inc_ref(x_90); lean_dec(x_89); lean_ctor_set(x_87, 1, x_90); -x_11 = x_79; -x_12 = x_81; -x_13 = lean_box(0); -x_14 = x_78; -x_15 = x_82; -x_16 = x_83; -x_17 = x_80; +x_11 = x_82; +x_12 = lean_box(0); +x_13 = x_78; +x_14 = x_81; +x_15 = x_80; +x_16 = x_79; +x_17 = x_83; x_18 = x_1; goto block_77; } @@ -7154,13 +7154,13 @@ x_94 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_94, 0, x_92); lean_ctor_set(x_94, 1, x_93); lean_ctor_set(x_1, 0, x_94); -x_11 = x_79; -x_12 = x_81; -x_13 = lean_box(0); -x_14 = x_78; -x_15 = x_82; -x_16 = x_83; -x_17 = x_80; +x_11 = x_82; +x_12 = lean_box(0); +x_13 = x_78; +x_14 = x_81; +x_15 = x_80; +x_16 = x_79; +x_17 = x_83; x_18 = x_1; goto block_77; } @@ -7195,13 +7195,13 @@ lean_ctor_set(x_100, 0, x_97); lean_ctor_set(x_100, 1, x_99); x_101 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_101, 0, x_100); -x_11 = x_79; -x_12 = x_81; -x_13 = lean_box(0); -x_14 = x_78; -x_15 = x_82; -x_16 = x_83; -x_17 = x_80; +x_11 = x_82; +x_12 = lean_box(0); +x_13 = x_78; +x_14 = x_81; +x_15 = x_80; +x_16 = x_79; +x_17 = x_83; x_18 = x_101; goto block_77; } @@ -9242,7 +9242,7 @@ goto block_47; { if (x_14 == 0) { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { lean_object* x_15; lean_dec(x_11); @@ -9271,7 +9271,7 @@ lean_object* x_20; lean_object* x_21; x_20 = lean_ctor_get(x_18, 0); lean_dec(x_20); x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_16); lean_ctor_set(x_18, 0, x_21); return x_18; @@ -9281,7 +9281,7 @@ else lean_object* x_22; lean_object* x_23; lean_dec(x_18); x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_12); +lean_ctor_set(x_22, 0, x_13); lean_ctor_set(x_22, 1, x_16); x_23 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_23, 0, x_22); @@ -9292,7 +9292,7 @@ else { uint8_t x_24; lean_dec(x_16); -lean_dec_ref(x_12); +lean_dec_ref(x_13); x_24 = !lean_is_exclusive(x_18); if (x_24 == 0) { @@ -9313,7 +9313,7 @@ return x_26; else { uint8_t x_27; -lean_dec_ref(x_12); +lean_dec_ref(x_13); lean_dec(x_10); lean_dec(x_7); lean_dec_ref(x_6); @@ -9341,7 +9341,7 @@ return x_29; else { lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_12, 0); +x_30 = lean_ctor_get(x_13, 0); x_31 = l_Lean_Elab_Term_observing___redArg___closed__0; x_32 = l_Lean_instBEqInternalExceptionId_beq(x_30, x_31); if (x_32 == 0) @@ -9360,7 +9360,7 @@ if (lean_is_scalar(x_11)) { x_33 = x_11; lean_ctor_set_tag(x_33, 1); } -lean_ctor_set(x_33, 0, x_12); +lean_ctor_set(x_33, 0, x_13); return x_33; } else @@ -9384,7 +9384,7 @@ lean_object* x_36; x_36 = lean_ctor_get(x_34, 0); lean_dec(x_36); lean_ctor_set_tag(x_34, 1); -lean_ctor_set(x_34, 0, x_12); +lean_ctor_set(x_34, 0, x_13); return x_34; } else @@ -9392,14 +9392,14 @@ else lean_object* x_37; lean_dec(x_34); x_37 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_37, 0, x_12); +lean_ctor_set(x_37, 0, x_13); return x_37; } } else { uint8_t x_38; -lean_dec_ref(x_12); +lean_dec_ref(x_13); x_38 = !lean_is_exclusive(x_34); if (x_38 == 0) { @@ -9435,7 +9435,7 @@ if (lean_is_scalar(x_11)) { x_41 = x_11; lean_ctor_set_tag(x_41, 1); } -lean_ctor_set(x_41, 0, x_12); +lean_ctor_set(x_41, 0, x_13); return x_41; } } @@ -9448,15 +9448,15 @@ if (x_45 == 0) uint8_t x_46; lean_inc_ref(x_43); x_46 = l_Lean_Exception_isRuntime(x_43); -x_12 = x_43; -x_13 = lean_box(0); +x_12 = lean_box(0); +x_13 = x_43; x_14 = x_46; goto block_42; } else { -x_12 = x_43; -x_13 = lean_box(0); +x_12 = lean_box(0); +x_13 = x_43; x_14 = x_45; goto block_42; } @@ -20416,7 +20416,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_logErrorAt___at___00Lean_Elab_Term_MVarErrorInfo_logError_spec__1_spec__1___redArg(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) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t 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_50; lean_object* x_51; uint8_t x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; uint8_t x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; uint8_t x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +lean_object* x_10; lean_object* x_11; uint8_t x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; uint8_t x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; uint8_t x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -20451,14 +20451,14 @@ lean_ctor_set(x_25, 0, x_21); lean_ctor_set(x_25, 1, x_22); x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_10); +lean_ctor_set(x_26, 1, x_16); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_15); -lean_ctor_set(x_27, 1, x_14); -lean_ctor_set(x_27, 2, x_13); -lean_ctor_set(x_27, 3, x_11); +lean_ctor_set(x_27, 0, x_14); +lean_ctor_set(x_27, 1, x_11); +lean_ctor_set(x_27, 2, x_10); +lean_ctor_set(x_27, 3, x_15); lean_ctor_set(x_27, 4, x_26); -lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_16); +lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_13); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_12); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); @@ -20496,14 +20496,14 @@ lean_ctor_set(x_41, 0, x_21); lean_ctor_set(x_41, 1, x_22); x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_10); +lean_ctor_set(x_42, 1, x_16); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_15); -lean_ctor_set(x_43, 1, x_14); -lean_ctor_set(x_43, 2, x_13); -lean_ctor_set(x_43, 3, x_11); +lean_ctor_set(x_43, 0, x_14); +lean_ctor_set(x_43, 1, x_11); +lean_ctor_set(x_43, 2, x_10); +lean_ctor_set(x_43, 3, x_15); lean_ctor_set(x_43, 4, x_42); -lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_16); +lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_13); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_12); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); @@ -20534,25 +20534,25 @@ if (x_60 == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); -lean_inc_ref(x_51); -x_62 = l_Lean_FileMap_toPosition(x_51, x_55); -lean_dec(x_55); -x_63 = l_Lean_FileMap_toPosition(x_51, x_57); +lean_inc_ref(x_52); +x_62 = l_Lean_FileMap_toPosition(x_52, x_51); +lean_dec(x_51); +x_63 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); x_65 = l_Lean_addTrace___at___00Lean_Elab_Term_traceAtCmdPos_spec__1___redArg___closed__1; -if (x_52 == 0) +if (x_56 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); -x_10 = x_61; -x_11 = x_65; +x_10 = x_64; +x_11 = x_62; x_12 = x_53; -x_13 = x_64; -x_14 = x_62; -x_15 = x_54; -x_16 = x_56; +x_13 = x_55; +x_14 = x_54; +x_15 = x_65; +x_16 = x_61; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -20578,13 +20578,13 @@ return x_59; else { lean_free_object(x_59); -x_10 = x_61; -x_11 = x_65; +x_10 = x_64; +x_11 = x_62; x_12 = x_53; -x_13 = x_64; -x_14 = x_62; -x_15 = x_54; -x_16 = x_56; +x_13 = x_55; +x_14 = x_54; +x_15 = x_65; +x_16 = x_61; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -20598,24 +20598,24 @@ lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); -lean_inc_ref(x_51); -x_69 = l_Lean_FileMap_toPosition(x_51, x_55); -lean_dec(x_55); -x_70 = l_Lean_FileMap_toPosition(x_51, x_57); +lean_inc_ref(x_52); +x_69 = l_Lean_FileMap_toPosition(x_52, x_51); +lean_dec(x_51); +x_70 = l_Lean_FileMap_toPosition(x_52, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); x_72 = l_Lean_addTrace___at___00Lean_Elab_Term_traceAtCmdPos_spec__1___redArg___closed__1; -if (x_52 == 0) +if (x_56 == 0) { lean_dec_ref(x_50); -x_10 = x_68; -x_11 = x_72; +x_10 = x_71; +x_11 = x_69; x_12 = x_53; -x_13 = x_71; -x_14 = x_69; -x_15 = x_54; -x_16 = x_56; +x_13 = x_55; +x_14 = x_54; +x_15 = x_72; +x_16 = x_68; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -20641,13 +20641,13 @@ return x_75; } else { -x_10 = x_68; -x_11 = x_72; +x_10 = x_71; +x_11 = x_69; x_12 = x_53; -x_13 = x_71; -x_14 = x_69; -x_15 = x_54; -x_16 = x_56; +x_13 = x_55; +x_14 = x_54; +x_15 = x_72; +x_16 = x_68; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -20659,17 +20659,17 @@ goto block_49; block_87: { lean_object* x_85; -x_85 = l_Lean_Syntax_getTailPos_x3f(x_78, x_83); +x_85 = l_Lean_Syntax_getTailPos_x3f(x_78, x_81); lean_dec(x_78); if (lean_obj_tag(x_85) == 0) { lean_inc(x_84); x_50 = x_77; -x_51 = x_79; -x_52 = x_80; -x_53 = x_81; +x_51 = x_84; +x_52 = x_79; +x_53 = x_80; x_54 = x_82; -x_55 = x_84; +x_55 = x_81; x_56 = x_83; x_57 = x_84; goto block_76; @@ -20681,11 +20681,11 @@ x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); lean_dec_ref(x_85); x_50 = x_77; -x_51 = x_79; -x_52 = x_80; -x_53 = x_81; +x_51 = x_84; +x_52 = x_79; +x_53 = x_80; x_54 = x_82; -x_55 = x_84; +x_55 = x_81; x_56 = x_83; x_57 = x_86; goto block_76; @@ -20694,8 +20694,8 @@ goto block_76; block_99: { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_replaceRef(x_1, x_93); -lean_dec(x_93); +x_95 = l_Lean_replaceRef(x_1, x_90); +lean_dec(x_90); x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_92); if (lean_obj_tag(x_96) == 0) { @@ -20704,10 +20704,10 @@ x_97 = lean_unsigned_to_nat(0u); x_77 = x_88; x_78 = x_95; x_79 = x_89; -x_80 = x_90; -x_81 = x_94; +x_80 = x_94; +x_81 = x_92; x_82 = x_91; -x_83 = x_92; +x_83 = x_93; x_84 = x_97; goto block_87; } @@ -20720,10 +20720,10 @@ lean_dec_ref(x_96); x_77 = x_88; x_78 = x_95; x_79 = x_89; -x_80 = x_90; -x_81 = x_94; +x_80 = x_94; +x_81 = x_92; x_82 = x_91; -x_83 = x_92; +x_83 = x_93; x_84 = x_98; goto block_87; } @@ -20732,10 +20732,10 @@ goto block_87; { if (x_107 == 0) { -x_88 = x_104; +x_88 = x_103; x_89 = x_101; x_90 = x_102; -x_91 = x_103; +x_91 = x_104; x_92 = x_106; x_93 = x_105; x_94 = x_3; @@ -20743,10 +20743,10 @@ goto block_99; } else { -x_88 = x_104; +x_88 = x_103; x_89 = x_101; x_90 = x_102; -x_91 = x_103; +x_91 = x_104; x_92 = x_106; x_93 = x_105; x_94 = x_100; @@ -20772,14 +20772,14 @@ x_118 = 1; x_119 = l_Lean_instBEqMessageSeverity_beq(x_3, x_118); if (x_119 == 0) { -lean_inc(x_113); lean_inc_ref(x_110); +lean_inc(x_113); lean_inc_ref(x_111); x_101 = x_111; -x_102 = x_114; -x_103 = x_110; -x_104 = x_117; -x_105 = x_113; +x_102 = x_113; +x_103 = x_117; +x_104 = x_110; +x_105 = x_114; x_106 = x_109; x_107 = x_119; goto block_108; @@ -20789,14 +20789,14 @@ else lean_object* x_120; uint8_t x_121; x_120 = l_Lean_logAt___at___00Lean_logErrorAt___at___00Lean_Elab_Term_MVarErrorInfo_logError_spec__1_spec__1___redArg___closed__0; x_121 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Elab_Term_throwErrorIfErrors_spec__0_spec__1_spec__2(x_112, x_120); -lean_inc(x_113); lean_inc_ref(x_110); +lean_inc(x_113); lean_inc_ref(x_111); x_101 = x_111; -x_102 = x_114; -x_103 = x_110; -x_104 = x_117; -x_105 = x_113; +x_102 = x_113; +x_103 = x_117; +x_104 = x_110; +x_105 = x_114; x_106 = x_109; x_107 = x_121; goto block_108; @@ -23542,7 +23542,7 @@ return x_18; LEAN_EXPORT lean_object* l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1___lam__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_10; 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; uint8_t x_18; 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_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_56; +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; uint8_t x_18; uint8_t 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_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; lean_object* x_56; lean_inc_ref(x_1); lean_inc(x_8); lean_inc_ref(x_7); @@ -23683,12 +23683,12 @@ x_69 = lean_ptr_addr(x_65); x_70 = lean_usize_dec_eq(x_68, x_69); if (x_70 == 0) { -x_42 = x_63; -x_43 = x_59; +x_42 = x_59; +x_43 = x_60; x_44 = lean_box(0); -x_45 = x_67; -x_46 = x_60; -x_47 = x_65; +x_45 = x_65; +x_46 = x_63; +x_47 = x_67; x_48 = x_70; goto block_55; } @@ -23698,12 +23698,12 @@ size_t x_71; size_t x_72; uint8_t x_73; x_71 = lean_ptr_addr(x_62); x_72 = lean_ptr_addr(x_67); x_73 = lean_usize_dec_eq(x_71, x_72); -x_42 = x_63; -x_43 = x_59; +x_42 = x_59; +x_43 = x_60; x_44 = lean_box(0); -x_45 = x_67; -x_46 = x_60; -x_47 = x_65; +x_45 = x_65; +x_46 = x_63; +x_47 = x_67; x_48 = x_73; goto block_55; } @@ -23780,12 +23780,12 @@ x_83 = lean_ptr_addr(x_79); x_84 = lean_usize_dec_eq(x_82, x_83); if (x_84 == 0) { -x_28 = x_74; -x_29 = x_81; -x_30 = lean_box(0); -x_31 = x_79; -x_32 = x_59; -x_33 = x_77; +x_28 = x_77; +x_29 = x_59; +x_30 = x_79; +x_31 = x_81; +x_32 = lean_box(0); +x_33 = x_74; x_34 = x_84; goto block_41; } @@ -23795,12 +23795,12 @@ size_t x_85; size_t x_86; uint8_t x_87; x_85 = lean_ptr_addr(x_76); x_86 = lean_ptr_addr(x_81); x_87 = lean_usize_dec_eq(x_85, x_86); -x_28 = x_74; -x_29 = x_81; -x_30 = lean_box(0); -x_31 = x_79; -x_32 = x_59; -x_33 = x_77; +x_28 = x_77; +x_29 = x_59; +x_30 = x_79; +x_31 = x_81; +x_32 = lean_box(0); +x_33 = x_74; x_34 = x_87; goto block_41; } @@ -23894,14 +23894,14 @@ x_100 = lean_ptr_addr(x_94); x_101 = lean_usize_dec_eq(x_99, x_100); if (x_101 == 0) { -x_10 = x_96; -x_11 = x_88; -x_12 = x_98; -x_13 = lean_box(0); -x_14 = x_91; -x_15 = x_59; -x_16 = x_94; -x_17 = x_92; +x_10 = x_91; +x_11 = x_98; +x_12 = x_59; +x_13 = x_94; +x_14 = x_92; +x_15 = x_88; +x_16 = x_96; +x_17 = lean_box(0); x_18 = x_101; goto block_27; } @@ -23911,14 +23911,14 @@ size_t x_102; size_t x_103; uint8_t x_104; x_102 = lean_ptr_addr(x_90); x_103 = lean_ptr_addr(x_96); x_104 = lean_usize_dec_eq(x_102, x_103); -x_10 = x_96; -x_11 = x_88; -x_12 = x_98; -x_13 = lean_box(0); -x_14 = x_91; -x_15 = x_59; -x_16 = x_94; -x_17 = x_92; +x_10 = x_91; +x_11 = x_98; +x_12 = x_59; +x_13 = x_94; +x_14 = x_92; +x_15 = x_88; +x_16 = x_96; +x_17 = lean_box(0); x_18 = x_104; goto block_27; } @@ -24231,12 +24231,12 @@ x_152 = lean_ptr_addr(x_148); x_153 = lean_usize_dec_eq(x_151, x_152); if (x_153 == 0) { -x_42 = x_146; -x_43 = x_142; +x_42 = x_142; +x_43 = x_143; x_44 = lean_box(0); -x_45 = x_150; -x_46 = x_143; -x_47 = x_148; +x_45 = x_148; +x_46 = x_146; +x_47 = x_150; x_48 = x_153; goto block_55; } @@ -24246,12 +24246,12 @@ size_t x_154; size_t x_155; uint8_t x_156; x_154 = lean_ptr_addr(x_145); x_155 = lean_ptr_addr(x_150); x_156 = lean_usize_dec_eq(x_154, x_155); -x_42 = x_146; -x_43 = x_142; +x_42 = x_142; +x_43 = x_143; x_44 = lean_box(0); -x_45 = x_150; -x_46 = x_143; -x_47 = x_148; +x_45 = x_148; +x_46 = x_146; +x_47 = x_150; x_48 = x_156; goto block_55; } @@ -24328,12 +24328,12 @@ x_166 = lean_ptr_addr(x_162); x_167 = lean_usize_dec_eq(x_165, x_166); if (x_167 == 0) { -x_28 = x_157; -x_29 = x_164; -x_30 = lean_box(0); -x_31 = x_162; -x_32 = x_142; -x_33 = x_160; +x_28 = x_160; +x_29 = x_142; +x_30 = x_162; +x_31 = x_164; +x_32 = lean_box(0); +x_33 = x_157; x_34 = x_167; goto block_41; } @@ -24343,12 +24343,12 @@ size_t x_168; size_t x_169; uint8_t x_170; x_168 = lean_ptr_addr(x_159); x_169 = lean_ptr_addr(x_164); x_170 = lean_usize_dec_eq(x_168, x_169); -x_28 = x_157; -x_29 = x_164; -x_30 = lean_box(0); -x_31 = x_162; -x_32 = x_142; -x_33 = x_160; +x_28 = x_160; +x_29 = x_142; +x_30 = x_162; +x_31 = x_164; +x_32 = lean_box(0); +x_33 = x_157; x_34 = x_170; goto block_41; } @@ -24442,14 +24442,14 @@ x_183 = lean_ptr_addr(x_177); x_184 = lean_usize_dec_eq(x_182, x_183); if (x_184 == 0) { -x_10 = x_179; -x_11 = x_171; -x_12 = x_181; -x_13 = lean_box(0); -x_14 = x_174; -x_15 = x_142; -x_16 = x_177; -x_17 = x_175; +x_10 = x_174; +x_11 = x_181; +x_12 = x_142; +x_13 = x_177; +x_14 = x_175; +x_15 = x_171; +x_16 = x_179; +x_17 = lean_box(0); x_18 = x_184; goto block_27; } @@ -24459,14 +24459,14 @@ size_t x_185; size_t x_186; uint8_t x_187; x_185 = lean_ptr_addr(x_173); x_186 = lean_ptr_addr(x_179); x_187 = lean_usize_dec_eq(x_185, x_186); -x_10 = x_179; -x_11 = x_171; -x_12 = x_181; -x_13 = lean_box(0); -x_14 = x_174; -x_15 = x_142; -x_16 = x_177; -x_17 = x_175; +x_10 = x_174; +x_11 = x_181; +x_12 = x_142; +x_13 = x_177; +x_14 = x_175; +x_15 = x_171; +x_16 = x_179; +x_17 = lean_box(0); x_18 = x_187; goto block_27; } @@ -24682,24 +24682,24 @@ return x_227; if (x_18 == 0) { lean_object* x_19; lean_object* x_20; -lean_dec_ref(x_15); -lean_dec_ref(x_14); -x_19 = l_Lean_Expr_letE___override(x_11, x_16, x_10, x_12, x_17); +lean_dec_ref(x_12); +lean_dec_ref(x_10); +x_19 = l_Lean_Expr_letE___override(x_15, x_13, x_16, x_11, x_14); x_20 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_19, x_4, x_5, x_6, x_7, x_8); return x_20; } else { size_t x_21; size_t x_22; uint8_t x_23; -x_21 = lean_ptr_addr(x_14); -lean_dec_ref(x_14); -x_22 = lean_ptr_addr(x_12); +x_21 = lean_ptr_addr(x_10); +lean_dec_ref(x_10); +x_22 = lean_ptr_addr(x_11); x_23 = lean_usize_dec_eq(x_21, x_22); if (x_23 == 0) { lean_object* x_24; lean_object* x_25; -lean_dec_ref(x_15); -x_24 = l_Lean_Expr_letE___override(x_11, x_16, x_10, x_12, x_17); +lean_dec_ref(x_12); +x_24 = l_Lean_Expr_letE___override(x_15, x_13, x_16, x_11, x_14); x_25 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_24, x_4, x_5, x_6, x_7, x_8); return x_25; } @@ -24707,10 +24707,10 @@ else { lean_object* x_26; lean_dec_ref(x_16); -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_10); -x_26 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_15, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_15); +lean_dec_ref(x_13); +lean_dec_ref(x_11); +x_26 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_12, x_4, x_5, x_6, x_7, x_8); return x_26; } } @@ -24720,30 +24720,30 @@ return x_26; if (x_34 == 0) { lean_object* x_35; lean_object* x_36; -lean_dec_ref(x_32); -x_35 = l_Lean_Expr_lam___override(x_28, x_31, x_29, x_33); +lean_dec_ref(x_29); +x_35 = l_Lean_Expr_lam___override(x_33, x_30, x_31, x_28); x_36 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_35, x_4, x_5, x_6, x_7, x_8); return x_36; } else { uint8_t x_37; -x_37 = l_Lean_instBEqBinderInfo_beq(x_33, x_33); +x_37 = l_Lean_instBEqBinderInfo_beq(x_28, x_28); if (x_37 == 0) { lean_object* x_38; lean_object* x_39; -lean_dec_ref(x_32); -x_38 = l_Lean_Expr_lam___override(x_28, x_31, x_29, x_33); +lean_dec_ref(x_29); +x_38 = l_Lean_Expr_lam___override(x_33, x_30, x_31, x_28); x_39 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_38, x_4, x_5, x_6, x_7, x_8); return x_39; } else { lean_object* x_40; +lean_dec(x_33); lean_dec_ref(x_31); -lean_dec_ref(x_29); -lean_dec(x_28); -x_40 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_32, x_4, x_5, x_6, x_7, x_8); +lean_dec_ref(x_30); +x_40 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_29, x_4, x_5, x_6, x_7, x_8); return x_40; } } @@ -24753,20 +24753,20 @@ return x_40; if (x_48 == 0) { lean_object* x_49; lean_object* x_50; -lean_dec_ref(x_43); -x_49 = l_Lean_Expr_forallE___override(x_46, x_47, x_45, x_42); +lean_dec_ref(x_42); +x_49 = l_Lean_Expr_forallE___override(x_43, x_45, x_47, x_46); x_50 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_49, x_4, x_5, x_6, x_7, x_8); return x_50; } else { uint8_t x_51; -x_51 = l_Lean_instBEqBinderInfo_beq(x_42, x_42); +x_51 = l_Lean_instBEqBinderInfo_beq(x_46, x_46); if (x_51 == 0) { lean_object* x_52; lean_object* x_53; -lean_dec_ref(x_43); -x_52 = l_Lean_Expr_forallE___override(x_46, x_47, x_45, x_42); +lean_dec_ref(x_42); +x_52 = l_Lean_Expr_forallE___override(x_43, x_45, x_47, x_46); x_53 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_52, x_4, x_5, x_6, x_7, x_8); return x_53; } @@ -24774,9 +24774,9 @@ else { lean_object* x_54; lean_dec_ref(x_47); -lean_dec(x_46); lean_dec_ref(x_45); -x_54 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_43, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_43); +x_54 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit_visitPost___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00Lean_Elab_Term_exposeLevelMVars_spec__1_spec__1_spec__3(x_1, x_3, x_42, x_4, x_5, x_6, x_7, x_8); return x_54; } } @@ -28821,7 +28821,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg(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_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_32; double x_33; double x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_43; double x_44; uint8_t x_45; double x_46; lean_object* x_47; lean_object* x_48; 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_70; double x_71; double x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_81; double x_82; lean_object* x_83; double x_84; lean_object* x_85; uint8_t x_86; lean_object* x_91; lean_object* x_92; lean_object* x_93; double x_94; double x_95; uint8_t x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; lean_object* x_133; double x_134; uint8_t x_135; double x_136; lean_object* x_137; lean_object* x_138; double x_139; lean_object* x_143; uint8_t x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_165; double x_166; double x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; uint8_t x_171; lean_object* x_205; double x_206; lean_object* x_207; double x_208; lean_object* x_209; uint8_t x_210; double x_211; uint8_t x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_255; +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_32; double x_33; uint8_t x_34; double x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_43; lean_object* x_44; uint8_t x_45; double x_46; lean_object* x_47; double x_48; 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; uint8_t x_70; double x_71; lean_object* x_72; double x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_81; double x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; double x_86; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; double x_95; uint8_t x_96; double x_97; lean_object* x_98; uint8_t x_99; lean_object* x_133; lean_object* x_134; uint8_t x_135; double x_136; lean_object* x_137; double x_138; double x_139; lean_object* x_143; lean_object* x_144; uint8_t x_145; lean_object* x_146; lean_object* x_147; uint8_t x_165; double x_166; lean_object* x_167; lean_object* x_168; double x_169; lean_object* x_170; uint8_t x_171; uint8_t x_205; double x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; double x_210; double x_211; lean_object* x_215; lean_object* x_216; uint8_t x_217; lean_object* x_218; lean_object* x_219; uint8_t x_255; x_13 = lean_ctor_get(x_10, 2); x_14 = lean_ctor_get(x_10, 5); lean_inc(x_1); @@ -28861,7 +28861,7 @@ goto block_254; lean_object* x_26; lean_dec(x_20); lean_dec_ref(x_19); -x_26 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__6___redArg(x_17, x_18, x_14, x_16, x_21, x_22, x_23, x_24); +x_26 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__6___redArg(x_15, x_18, x_14, x_16, x_21, x_22, x_23, x_24); lean_dec(x_24); lean_dec(x_22); lean_dec_ref(x_21); @@ -28869,13 +28869,13 @@ if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_dec_ref(x_26); -x_27 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_15); +x_27 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_17); return x_27; } else { uint8_t x_28; -lean_dec_ref(x_15); +lean_dec_ref(x_17); x_28 = !lean_is_exclusive(x_26); if (x_28 == 0) { @@ -28895,7 +28895,7 @@ return x_30; } block_42: { -if (x_35 == 0) +if (x_34 == 0) { double x_39; lean_object* x_40; x_39 = l_Lean_addTrace___at___00Lean_Elab_Term_traceAtCmdPos_spec__1___redArg___closed__0; @@ -28925,7 +28925,7 @@ x_41 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_41, 0, x_1); lean_ctor_set(x_41, 1, x_5); lean_ctor_set_float(x_41, sizeof(void*)*2, x_33); -lean_ctor_set_float(x_41, sizeof(void*)*2 + 8, x_34); +lean_ctor_set_float(x_41, sizeof(void*)*2 + 8, x_35); lean_ctor_set_uint8(x_41, sizeof(void*)*2 + 16, x_4); x_15 = x_32; x_16 = x_37; @@ -28950,19 +28950,19 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_43); -x_49 = lean_apply_8(x_2, x_43, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); +lean_inc_ref(x_47); +x_49 = lean_apply_8(x_2, x_47, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_49) == 0) { lean_object* x_50; x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); lean_dec_ref(x_49); -x_32 = x_43; -x_33 = x_44; -x_34 = x_46; -x_35 = x_45; -x_36 = x_48; +x_32 = x_44; +x_33 = x_46; +x_34 = x_45; +x_35 = x_48; +x_36 = x_47; x_37 = x_50; x_38 = lean_box(0); goto block_42; @@ -28972,11 +28972,11 @@ else lean_object* x_51; lean_dec_ref(x_49); x_51 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__1; -x_32 = x_43; -x_33 = x_44; -x_34 = x_46; -x_35 = x_45; -x_36 = x_48; +x_32 = x_44; +x_33 = x_46; +x_34 = x_45; +x_35 = x_48; +x_36 = x_47; x_37 = x_51; x_38 = lean_box(0); goto block_42; @@ -28987,7 +28987,7 @@ goto block_42; lean_object* x_64; lean_dec(x_58); lean_dec_ref(x_57); -x_64 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__6___redArg(x_55, x_56, x_14, x_54, x_59, x_60, x_61, x_62); +x_64 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__6___redArg(x_54, x_56, x_14, x_53, x_59, x_60, x_61, x_62); lean_dec(x_62); lean_dec(x_60); lean_dec_ref(x_59); @@ -28995,13 +28995,13 @@ if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_dec_ref(x_64); -x_65 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_53); +x_65 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_55); return x_65; } else { uint8_t x_66; -lean_dec_ref(x_53); +lean_dec_ref(x_55); x_66 = !lean_is_exclusive(x_64); if (x_66 == 0) { @@ -29021,7 +29021,7 @@ return x_68; } block_80: { -if (x_74 == 0) +if (x_70 == 0) { double x_77; lean_object* x_78; x_77 = l_Lean_addTrace___at___00Lean_Elab_Term_traceAtCmdPos_spec__1___redArg___closed__0; @@ -29031,9 +29031,9 @@ lean_ctor_set(x_78, 1, x_5); lean_ctor_set_float(x_78, sizeof(void*)*2, x_77); lean_ctor_set_float(x_78, sizeof(void*)*2 + 8, x_77); lean_ctor_set_uint8(x_78, sizeof(void*)*2 + 16, x_4); -x_53 = x_70; -x_54 = x_75; -x_55 = x_73; +x_53 = x_75; +x_54 = x_72; +x_55 = x_74; x_56 = x_78; x_57 = x_6; x_58 = x_7; @@ -29050,12 +29050,12 @@ lean_object* x_79; x_79 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_79, 0, x_1); lean_ctor_set(x_79, 1, x_5); -lean_ctor_set_float(x_79, sizeof(void*)*2, x_71); -lean_ctor_set_float(x_79, sizeof(void*)*2 + 8, x_72); +lean_ctor_set_float(x_79, sizeof(void*)*2, x_73); +lean_ctor_set_float(x_79, sizeof(void*)*2 + 8, x_71); lean_ctor_set_uint8(x_79, sizeof(void*)*2 + 16, x_4); -x_53 = x_70; -x_54 = x_75; -x_55 = x_73; +x_53 = x_75; +x_54 = x_72; +x_55 = x_74; x_56 = x_79; x_57 = x_6; x_58 = x_7; @@ -29076,8 +29076,8 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_81); -x_87 = lean_apply_8(x_2, x_81, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); +lean_inc_ref(x_85); +x_87 = lean_apply_8(x_2, x_85, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_87) == 0) { lean_object* x_88; @@ -29086,9 +29086,9 @@ lean_inc(x_88); lean_dec_ref(x_87); x_70 = x_81; x_71 = x_82; -x_72 = x_84; -x_73 = x_85; -x_74 = x_86; +x_72 = x_83; +x_73 = x_86; +x_74 = x_85; x_75 = x_88; x_76 = lean_box(0); goto block_80; @@ -29100,9 +29100,9 @@ lean_dec_ref(x_87); x_89 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__1; x_70 = x_81; x_71 = x_82; -x_72 = x_84; -x_73 = x_85; -x_74 = x_86; +x_72 = x_83; +x_73 = x_86; +x_74 = x_85; x_75 = x_89; x_76 = lean_box(0); goto block_80; @@ -29138,12 +29138,12 @@ if (x_104 == 0) { lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; x_105 = lean_ctor_get(x_103, 0); -x_106 = l_Lean_PersistentArray_append___redArg(x_97, x_105); +x_106 = l_Lean_PersistentArray_append___redArg(x_94, x_105); lean_dec_ref(x_105); lean_ctor_set(x_103, 0, x_106); x_107 = lean_st_ref_set(x_11, x_101); lean_dec(x_11); -x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_93); +x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_98); return x_108; } else @@ -29153,7 +29153,7 @@ x_109 = lean_ctor_get_uint64(x_103, sizeof(void*)*1); x_110 = lean_ctor_get(x_103, 0); lean_inc(x_110); lean_dec(x_103); -x_111 = l_Lean_PersistentArray_append___redArg(x_97, x_110); +x_111 = l_Lean_PersistentArray_append___redArg(x_94, x_110); lean_dec_ref(x_110); x_112 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_112, 0, x_111); @@ -29161,7 +29161,7 @@ lean_ctor_set_uint64(x_112, sizeof(void*)*1, x_109); lean_ctor_set(x_101, 4, x_112); x_113 = lean_st_ref_set(x_11, x_101); lean_dec(x_11); -x_114 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_93); +x_114 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_98); return x_114; } } @@ -29197,7 +29197,7 @@ if (lean_is_exclusive(x_115)) { lean_dec_ref(x_115); x_126 = lean_box(0); } -x_127 = l_Lean_PersistentArray_append___redArg(x_97, x_125); +x_127 = l_Lean_PersistentArray_append___redArg(x_94, x_125); lean_dec_ref(x_125); if (lean_is_scalar(x_126)) { x_128 = lean_alloc_ctor(0, 1, 8); @@ -29218,28 +29218,28 @@ lean_ctor_set(x_129, 7, x_122); lean_ctor_set(x_129, 8, x_123); x_130 = lean_st_ref_set(x_11, x_129); lean_dec(x_11); -x_131 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_93); +x_131 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_98); return x_131; } } else { -x_43 = x_93; +x_43 = lean_box(0); x_44 = x_94; x_45 = x_96; x_46 = x_95; -x_47 = lean_box(0); +x_47 = x_98; x_48 = x_97; goto block_52; } } else { -x_43 = x_93; +x_43 = lean_box(0); x_44 = x_94; x_45 = x_96; x_46 = x_95; -x_47 = lean_box(0); +x_47 = x_98; x_48 = x_97; goto block_52; } @@ -29247,14 +29247,14 @@ goto block_52; block_142: { double x_140; uint8_t x_141; -x_140 = lean_float_sub(x_136, x_134); +x_140 = lean_float_sub(x_138, x_136); x_141 = lean_float_decLt(x_139, x_140); -x_93 = x_133; +x_93 = lean_box(0); x_94 = x_134; x_95 = x_136; x_96 = x_135; x_97 = x_138; -x_98 = lean_box(0); +x_98 = x_137; x_99 = x_141; goto block_132; } @@ -29262,7 +29262,7 @@ goto block_132; { lean_object* x_148; double x_149; double x_150; double x_151; double x_152; double x_153; lean_object* x_154; uint8_t x_155; x_148 = lean_io_mono_nanos_now(); -x_149 = lean_float_of_nat(x_143); +x_149 = lean_float_of_nat(x_144); x_150 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__2; x_151 = lean_float_div(x_149, x_150); x_152 = lean_float_of_nat(x_148); @@ -29271,18 +29271,18 @@ x_154 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean x_155 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Elab_Term_throwErrorIfErrors_spec__0_spec__1_spec__2(x_13, x_154); if (x_155 == 0) { -x_93 = x_146; -x_94 = x_151; -x_95 = x_153; +x_93 = lean_box(0); +x_94 = x_143; +x_95 = x_151; x_96 = x_155; -x_97 = x_145; -x_98 = lean_box(0); +x_97 = x_153; +x_98 = x_146; x_99 = x_155; goto block_132; } else { -if (x_144 == 0) +if (x_145 == 0) { lean_object* x_156; lean_object* x_157; double x_158; double x_159; double x_160; x_156 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; @@ -29290,12 +29290,12 @@ x_157 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_El x_158 = lean_float_of_nat(x_157); x_159 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__5; x_160 = lean_float_div(x_158, x_159); -x_133 = x_146; -x_134 = x_151; +x_133 = lean_box(0); +x_134 = x_143; x_135 = x_155; -x_136 = x_153; -x_137 = lean_box(0); -x_138 = x_145; +x_136 = x_151; +x_137 = x_146; +x_138 = x_153; x_139 = x_160; goto block_142; } @@ -29305,12 +29305,12 @@ lean_object* x_161; lean_object* x_162; double x_163; x_161 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; x_162 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__8(x_13, x_161); x_163 = lean_float_of_nat(x_162); -x_133 = x_146; -x_134 = x_151; +x_133 = lean_box(0); +x_134 = x_143; x_135 = x_155; -x_136 = x_153; -x_137 = lean_box(0); -x_138 = x_145; +x_136 = x_151; +x_137 = x_146; +x_138 = x_153; x_139 = x_163; goto block_142; } @@ -29346,12 +29346,12 @@ if (x_176 == 0) { lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; x_177 = lean_ctor_get(x_175, 0); -x_178 = l_Lean_PersistentArray_append___redArg(x_169, x_177); +x_178 = l_Lean_PersistentArray_append___redArg(x_167, x_177); lean_dec_ref(x_177); lean_ctor_set(x_175, 0, x_178); x_179 = lean_st_ref_set(x_11, x_173); lean_dec(x_11); -x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_165); +x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_180; } else @@ -29361,7 +29361,7 @@ x_181 = lean_ctor_get_uint64(x_175, sizeof(void*)*1); x_182 = lean_ctor_get(x_175, 0); lean_inc(x_182); lean_dec(x_175); -x_183 = l_Lean_PersistentArray_append___redArg(x_169, x_182); +x_183 = l_Lean_PersistentArray_append___redArg(x_167, x_182); lean_dec_ref(x_182); x_184 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_184, 0, x_183); @@ -29369,7 +29369,7 @@ lean_ctor_set_uint64(x_184, sizeof(void*)*1, x_181); lean_ctor_set(x_173, 4, x_184); x_185 = lean_st_ref_set(x_11, x_173); lean_dec(x_11); -x_186 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_165); +x_186 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_186; } } @@ -29405,7 +29405,7 @@ if (lean_is_exclusive(x_187)) { lean_dec_ref(x_187); x_198 = lean_box(0); } -x_199 = l_Lean_PersistentArray_append___redArg(x_169, x_197); +x_199 = l_Lean_PersistentArray_append___redArg(x_167, x_197); lean_dec_ref(x_197); if (lean_is_scalar(x_198)) { x_200 = lean_alloc_ctor(0, 1, 8); @@ -29426,7 +29426,7 @@ lean_ctor_set(x_201, 7, x_194); lean_ctor_set(x_201, 8, x_195); x_202 = lean_st_ref_set(x_11, x_201); lean_dec(x_11); -x_203 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_165); +x_203 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_203; } } @@ -29434,10 +29434,10 @@ else { x_81 = x_165; x_82 = x_166; -x_83 = lean_box(0); -x_84 = x_167; -x_85 = x_169; -x_86 = x_170; +x_83 = x_167; +x_84 = lean_box(0); +x_85 = x_170; +x_86 = x_169; goto block_90; } } @@ -29445,24 +29445,24 @@ else { x_81 = x_165; x_82 = x_166; -x_83 = lean_box(0); -x_84 = x_167; -x_85 = x_169; -x_86 = x_170; +x_83 = x_167; +x_84 = lean_box(0); +x_85 = x_170; +x_86 = x_169; goto block_90; } } block_214: { double x_212; uint8_t x_213; -x_212 = lean_float_sub(x_208, x_206); +x_212 = lean_float_sub(x_206, x_210); x_213 = lean_float_decLt(x_211, x_212); x_165 = x_205; x_166 = x_206; -x_167 = x_208; +x_167 = x_207; x_168 = lean_box(0); -x_169 = x_209; -x_170 = x_210; +x_169 = x_210; +x_170 = x_209; x_171 = x_213; goto block_204; } @@ -29470,24 +29470,24 @@ goto block_204; { lean_object* x_220; double x_221; double x_222; lean_object* x_223; uint8_t x_224; x_220 = lean_io_get_num_heartbeats(); -x_221 = lean_float_of_nat(x_217); +x_221 = lean_float_of_nat(x_215); x_222 = lean_float_of_nat(x_220); x_223 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__3; x_224 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Elab_Term_throwErrorIfErrors_spec__0_spec__1_spec__2(x_13, x_223); if (x_224 == 0) { -x_165 = x_218; -x_166 = x_221; -x_167 = x_222; +x_165 = x_224; +x_166 = x_222; +x_167 = x_216; x_168 = lean_box(0); -x_169 = x_216; -x_170 = x_224; +x_169 = x_221; +x_170 = x_218; x_171 = x_224; goto block_204; } else { -if (x_215 == 0) +if (x_217 == 0) { lean_object* x_225; lean_object* x_226; double x_227; double x_228; double x_229; x_225 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; @@ -29495,12 +29495,12 @@ x_226 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_El x_227 = lean_float_of_nat(x_226); x_228 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__5; x_229 = lean_float_div(x_227, x_228); -x_205 = x_218; -x_206 = x_221; -x_207 = lean_box(0); -x_208 = x_222; -x_209 = x_216; -x_210 = x_224; +x_205 = x_224; +x_206 = x_222; +x_207 = x_216; +x_208 = lean_box(0); +x_209 = x_218; +x_210 = x_221; x_211 = x_229; goto block_214; } @@ -29510,12 +29510,12 @@ lean_object* x_230; lean_object* x_231; double x_232; x_230 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; x_231 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__8(x_13, x_230); x_232 = lean_float_of_nat(x_231); -x_205 = x_218; -x_206 = x_221; -x_207 = lean_box(0); -x_208 = x_222; -x_209 = x_216; -x_210 = x_224; +x_205 = x_224; +x_206 = x_222; +x_207 = x_216; +x_208 = lean_box(0); +x_209 = x_218; +x_210 = x_221; x_211 = x_232; goto block_214; } @@ -29548,9 +29548,9 @@ x_240 = !lean_is_exclusive(x_239); if (x_240 == 0) { lean_ctor_set_tag(x_239, 1); -x_143 = x_238; -x_144 = x_237; -x_145 = x_235; +x_143 = x_235; +x_144 = x_238; +x_145 = x_237; x_146 = x_239; x_147 = lean_box(0); goto block_164; @@ -29563,9 +29563,9 @@ lean_inc(x_241); lean_dec(x_239); x_242 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_242, 0, x_241); -x_143 = x_238; -x_144 = x_237; -x_145 = x_235; +x_143 = x_235; +x_144 = x_238; +x_145 = x_237; x_146 = x_242; x_147 = lean_box(0); goto block_164; @@ -29578,9 +29578,9 @@ x_243 = !lean_is_exclusive(x_239); if (x_243 == 0) { lean_ctor_set_tag(x_239, 0); -x_143 = x_238; -x_144 = x_237; -x_145 = x_235; +x_143 = x_235; +x_144 = x_238; +x_145 = x_237; x_146 = x_239; x_147 = lean_box(0); goto block_164; @@ -29593,9 +29593,9 @@ lean_inc(x_244); lean_dec(x_239); x_245 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_245, 0, x_244); -x_143 = x_238; -x_144 = x_237; -x_145 = x_235; +x_143 = x_235; +x_144 = x_238; +x_145 = x_237; x_146 = x_245; x_147 = lean_box(0); goto block_164; @@ -29620,9 +29620,9 @@ x_248 = !lean_is_exclusive(x_247); if (x_248 == 0) { lean_ctor_set_tag(x_247, 1); -x_215 = x_237; +x_215 = x_246; x_216 = x_235; -x_217 = x_246; +x_217 = x_237; x_218 = x_247; x_219 = lean_box(0); goto block_233; @@ -29635,9 +29635,9 @@ lean_inc(x_249); lean_dec(x_247); x_250 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_250, 0, x_249); -x_215 = x_237; +x_215 = x_246; x_216 = x_235; -x_217 = x_246; +x_217 = x_237; x_218 = x_250; x_219 = lean_box(0); goto block_233; @@ -29650,9 +29650,9 @@ x_251 = !lean_is_exclusive(x_247); if (x_251 == 0) { lean_ctor_set_tag(x_247, 0); -x_215 = x_237; +x_215 = x_246; x_216 = x_235; -x_217 = x_246; +x_217 = x_237; x_218 = x_247; x_219 = lean_box(0); goto block_233; @@ -29665,9 +29665,9 @@ lean_inc(x_252); lean_dec(x_247); x_253 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_253, 0, x_252); -x_215 = x_237; +x_215 = x_246; x_216 = x_235; -x_217 = x_246; +x_217 = x_237; x_218 = x_253; x_219 = lean_box(0); goto block_233; @@ -40842,7 +40842,7 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_27; uint8_t x_37; +lean_object* x_14; uint8_t x_15; lean_object* x_16; uint8_t x_27; uint8_t x_37; x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_37 = l_Lean_Exception_isInterrupt(x_14); @@ -40863,12 +40863,12 @@ goto block_36; { lean_object* x_17; uint8_t x_18; x_17 = l_Lean_Elab_throwUnsupportedSyntax___at___00Lean_Elab_Term_elabFixedTermElab_spec__0___redArg___closed__0; -x_18 = l_Lean_instBEqInternalExceptionId_beq(x_15, x_17); +x_18 = l_Lean_instBEqInternalExceptionId_beq(x_16, x_17); if (x_18 == 0) { if (x_4 == 0) { -lean_dec(x_15); +lean_dec(x_16); lean_dec(x_11); lean_dec_ref(x_10); lean_dec(x_9); @@ -40884,8 +40884,8 @@ else { lean_object* x_19; uint8_t x_20; x_19 = l_Lean_Elab_Term_observing___redArg___closed__0; -x_20 = l_Lean_instBEqInternalExceptionId_beq(x_15, x_19); -lean_dec(x_15); +x_20 = l_Lean_instBEqInternalExceptionId_beq(x_16, x_19); +lean_dec(x_16); if (x_20 == 0) { lean_dec(x_11); @@ -40903,7 +40903,7 @@ else { lean_object* x_21; lean_dec_ref(x_13); -x_21 = l_Lean_Elab_Term_SavedState_restore(x_5, x_16, x_6, x_7, x_8, x_9, x_10, x_11); +x_21 = l_Lean_Elab_Term_SavedState_restore(x_5, x_15, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; @@ -40948,7 +40948,7 @@ return x_25; } else { -lean_dec(x_15); +lean_dec(x_16); lean_dec(x_11); lean_dec_ref(x_10); lean_dec(x_9); @@ -41003,8 +41003,8 @@ lean_object* x_31; x_31 = lean_ctor_get(x_14, 0); lean_inc(x_31); lean_dec_ref(x_14); -x_15 = x_31; -x_16 = x_27; +x_15 = x_27; +x_16 = x_31; goto block_26; } else @@ -41017,8 +41017,8 @@ if (x_34 == 0) { lean_inc(x_32); lean_dec_ref(x_14); -x_15 = x_32; -x_16 = x_27; +x_15 = x_27; +x_16 = x_32; goto block_26; } else @@ -43304,9 +43304,9 @@ goto block_59; { lean_object* x_23; x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_13); +lean_ctor_set(x_23, 0, x_14); lean_ctor_set(x_23, 1, x_4); -x_3 = x_14; +x_3 = x_13; x_4 = x_23; x_5 = x_15; x_6 = x_16; @@ -43353,8 +43353,8 @@ if (x_40 == 0) { uint8_t x_41; x_41 = 1; -x_13 = x_34; -x_14 = x_33; +x_13 = x_33; +x_14 = x_34; x_15 = x_41; x_16 = x_6; x_17 = x_7; @@ -43367,8 +43367,8 @@ goto block_25; } else { -x_13 = x_34; -x_14 = x_33; +x_13 = x_33; +x_14 = x_34; x_15 = x_5; x_16 = x_6; x_17 = x_7; @@ -43414,8 +43414,8 @@ lean_inc(x_45); x_46 = lean_ctor_get(x_3, 1); lean_inc_ref(x_46); lean_dec_ref(x_3); -x_13 = x_46; -x_14 = x_45; +x_13 = x_45; +x_14 = x_46; x_15 = x_5; x_16 = x_6; x_17 = x_7; @@ -47894,7 +47894,7 @@ return x_125; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_elabTermAux_spec__3___redArg(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_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; double x_32; lean_object* x_33; lean_object* x_34; double x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_43; double x_44; lean_object* x_45; lean_object* x_46; double x_47; uint8_t x_48; 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_70; lean_object* x_71; uint8_t x_72; double x_73; double x_74; lean_object* x_75; lean_object* x_76; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; double x_85; double x_86; lean_object* x_91; lean_object* x_92; lean_object* x_93; double x_94; lean_object* x_95; lean_object* x_96; double x_97; uint8_t x_98; uint8_t x_99; lean_object* x_133; double x_134; lean_object* x_135; lean_object* x_136; double x_137; uint8_t x_138; double x_139; lean_object* x_143; uint8_t x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_165; lean_object* x_166; lean_object* x_167; uint8_t x_168; double x_169; double x_170; uint8_t x_171; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; double x_209; double x_210; double x_211; uint8_t x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_255; +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; double x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; double x_36; lean_object* x_37; lean_object* x_38; lean_object* x_43; double x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; double x_48; 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; double x_70; double x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; double x_81; lean_object* x_82; double x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_91; lean_object* x_92; lean_object* x_93; double x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; double x_98; uint8_t x_99; lean_object* x_133; double x_134; lean_object* x_135; uint8_t x_136; lean_object* x_137; double x_138; double x_139; uint8_t x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; double x_165; double x_166; lean_object* x_167; uint8_t x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; double x_205; lean_object* x_206; double x_207; lean_object* x_208; uint8_t x_209; lean_object* x_210; double x_211; uint8_t x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_255; x_13 = lean_ctor_get(x_10, 2); x_14 = lean_ctor_get(x_10, 5); lean_inc(x_1); @@ -47934,7 +47934,7 @@ goto block_254; lean_object* x_26; lean_dec(x_20); lean_dec_ref(x_19); -x_26 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_elabTermAux_spec__3_spec__8___redArg(x_15, x_18, x_14, x_16, x_21, x_22, x_23, x_24); +x_26 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_elabTermAux_spec__3_spec__8___redArg(x_16, x_18, x_14, x_17, x_21, x_22, x_23, x_24); lean_dec(x_24); lean_dec(x_22); lean_dec_ref(x_21); @@ -47942,13 +47942,13 @@ if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_dec_ref(x_26); -x_27 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_17); +x_27 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_15); return x_27; } else { uint8_t x_28; -lean_dec_ref(x_17); +lean_dec_ref(x_15); x_28 = !lean_is_exclusive(x_26); if (x_28 == 0) { @@ -47968,7 +47968,7 @@ return x_30; } block_42: { -if (x_36 == 0) +if (x_34 == 0) { double x_39; lean_object* x_40; x_39 = l_Lean_addTrace___at___00Lean_Elab_Term_traceAtCmdPos_spec__1___redArg___closed__0; @@ -47979,8 +47979,8 @@ lean_ctor_set_float(x_40, sizeof(void*)*2, x_39); lean_ctor_set_float(x_40, sizeof(void*)*2 + 8, x_39); lean_ctor_set_uint8(x_40, sizeof(void*)*2 + 16, x_4); x_15 = x_33; -x_16 = x_37; -x_17 = x_34; +x_16 = x_35; +x_17 = x_37; x_18 = x_40; x_19 = x_6; x_20 = x_7; @@ -47997,12 +47997,12 @@ lean_object* x_41; x_41 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_41, 0, x_1); lean_ctor_set(x_41, 1, x_5); -lean_ctor_set_float(x_41, sizeof(void*)*2, x_35); +lean_ctor_set_float(x_41, sizeof(void*)*2, x_36); lean_ctor_set_float(x_41, sizeof(void*)*2 + 8, x_32); lean_ctor_set_uint8(x_41, sizeof(void*)*2 + 16, x_4); x_15 = x_33; -x_16 = x_37; -x_17 = x_34; +x_16 = x_35; +x_17 = x_37; x_18 = x_41; x_19 = x_6; x_20 = x_7; @@ -48023,8 +48023,8 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_46); -x_49 = lean_apply_8(x_2, x_46, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); +lean_inc_ref(x_45); +x_49 = lean_apply_8(x_2, x_45, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_49) == 0) { lean_object* x_50; @@ -48060,7 +48060,7 @@ goto block_42; lean_object* x_64; lean_dec(x_58); lean_dec_ref(x_57); -x_64 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_elabTermAux_spec__3_spec__8___redArg(x_53, x_56, x_14, x_55, x_59, x_60, x_61, x_62); +x_64 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_elabTermAux_spec__3_spec__8___redArg(x_54, x_56, x_14, x_53, x_59, x_60, x_61, x_62); lean_dec(x_62); lean_dec(x_60); lean_dec_ref(x_59); @@ -48068,13 +48068,13 @@ if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_dec_ref(x_64); -x_65 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_54); +x_65 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_55); return x_65; } else { uint8_t x_66; -lean_dec_ref(x_54); +lean_dec_ref(x_55); x_66 = !lean_is_exclusive(x_64); if (x_66 == 0) { @@ -48104,9 +48104,9 @@ lean_ctor_set(x_78, 1, x_5); lean_ctor_set_float(x_78, sizeof(void*)*2, x_77); lean_ctor_set_float(x_78, sizeof(void*)*2 + 8, x_77); lean_ctor_set_uint8(x_78, sizeof(void*)*2 + 16, x_4); -x_53 = x_70; -x_54 = x_71; -x_55 = x_75; +x_53 = x_75; +x_54 = x_73; +x_55 = x_74; x_56 = x_78; x_57 = x_6; x_58 = x_7; @@ -48123,12 +48123,12 @@ lean_object* x_79; x_79 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_79, 0, x_1); lean_ctor_set(x_79, 1, x_5); -lean_ctor_set_float(x_79, sizeof(void*)*2, x_74); -lean_ctor_set_float(x_79, sizeof(void*)*2 + 8, x_73); +lean_ctor_set_float(x_79, sizeof(void*)*2, x_70); +lean_ctor_set_float(x_79, sizeof(void*)*2 + 8, x_71); lean_ctor_set_uint8(x_79, sizeof(void*)*2 + 16, x_4); -x_53 = x_70; -x_54 = x_71; -x_55 = x_75; +x_53 = x_75; +x_54 = x_73; +x_55 = x_74; x_56 = x_79; x_57 = x_6; x_58 = x_7; @@ -48149,8 +48149,8 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_82); -x_87 = lean_apply_8(x_2, x_82, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); +lean_inc_ref(x_86); +x_87 = lean_apply_8(x_2, x_86, x_6, x_7, x_8, x_9, x_10, x_11, lean_box(0)); if (lean_obj_tag(x_87) == 0) { lean_object* x_88; @@ -48158,9 +48158,9 @@ x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); lean_dec_ref(x_87); x_70 = x_81; -x_71 = x_82; -x_72 = x_84; -x_73 = x_85; +x_71 = x_83; +x_72 = x_85; +x_73 = x_84; x_74 = x_86; x_75 = x_88; x_76 = lean_box(0); @@ -48172,9 +48172,9 @@ lean_object* x_89; lean_dec_ref(x_87); x_89 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__1; x_70 = x_81; -x_71 = x_82; -x_72 = x_84; -x_73 = x_85; +x_71 = x_83; +x_72 = x_85; +x_73 = x_84; x_74 = x_86; x_75 = x_89; x_76 = lean_box(0); @@ -48211,12 +48211,12 @@ if (x_104 == 0) { lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; x_105 = lean_ctor_get(x_103, 0); -x_106 = l_Lean_PersistentArray_append___redArg(x_95, x_105); +x_106 = l_Lean_PersistentArray_append___redArg(x_97, x_105); lean_dec_ref(x_105); lean_ctor_set(x_103, 0, x_106); x_107 = lean_st_ref_set(x_11, x_101); lean_dec(x_11); -x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_96); +x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_95); return x_108; } else @@ -48226,7 +48226,7 @@ x_109 = lean_ctor_get_uint64(x_103, sizeof(void*)*1); x_110 = lean_ctor_get(x_103, 0); lean_inc(x_110); lean_dec(x_103); -x_111 = l_Lean_PersistentArray_append___redArg(x_95, x_110); +x_111 = l_Lean_PersistentArray_append___redArg(x_97, x_110); lean_dec_ref(x_110); x_112 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_112, 0, x_111); @@ -48234,7 +48234,7 @@ lean_ctor_set_uint64(x_112, sizeof(void*)*1, x_109); lean_ctor_set(x_101, 4, x_112); x_113 = lean_st_ref_set(x_11, x_101); lean_dec(x_11); -x_114 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_96); +x_114 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_95); return x_114; } } @@ -48270,7 +48270,7 @@ if (lean_is_exclusive(x_115)) { lean_dec_ref(x_115); x_126 = lean_box(0); } -x_127 = l_Lean_PersistentArray_append___redArg(x_95, x_125); +x_127 = l_Lean_PersistentArray_append___redArg(x_97, x_125); lean_dec_ref(x_125); if (lean_is_scalar(x_126)) { x_128 = lean_alloc_ctor(0, 1, 8); @@ -48291,7 +48291,7 @@ lean_ctor_set(x_129, 7, x_122); lean_ctor_set(x_129, 8, x_123); x_130 = lean_st_ref_set(x_11, x_129); lean_dec(x_11); -x_131 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_96); +x_131 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_95); return x_131; } } @@ -48320,7 +48320,7 @@ goto block_52; block_142: { double x_140; uint8_t x_141; -x_140 = lean_float_sub(x_134, x_137); +x_140 = lean_float_sub(x_134, x_138); x_141 = lean_float_decLt(x_139, x_140); x_93 = lean_box(0); x_94 = x_134; @@ -48335,7 +48335,7 @@ goto block_132; { lean_object* x_148; double x_149; double x_150; double x_151; double x_152; double x_153; lean_object* x_154; uint8_t x_155; x_148 = lean_io_mono_nanos_now(); -x_149 = lean_float_of_nat(x_143); +x_149 = lean_float_of_nat(x_144); x_150 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__2; x_151 = lean_float_div(x_149, x_150); x_152 = lean_float_of_nat(x_148); @@ -48346,16 +48346,16 @@ if (x_155 == 0) { x_93 = lean_box(0); x_94 = x_153; -x_95 = x_145; -x_96 = x_146; -x_97 = x_151; -x_98 = x_155; +x_95 = x_146; +x_96 = x_155; +x_97 = x_145; +x_98 = x_151; x_99 = x_155; goto block_132; } else { -if (x_144 == 0) +if (x_143 == 0) { lean_object* x_156; lean_object* x_157; double x_158; double x_159; double x_160; x_156 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; @@ -48365,10 +48365,10 @@ x_159 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean x_160 = lean_float_div(x_158, x_159); x_133 = lean_box(0); x_134 = x_153; -x_135 = x_145; -x_136 = x_146; -x_137 = x_151; -x_138 = x_155; +x_135 = x_146; +x_136 = x_155; +x_137 = x_145; +x_138 = x_151; x_139 = x_160; goto block_142; } @@ -48380,10 +48380,10 @@ x_162 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_El x_163 = lean_float_of_nat(x_162); x_133 = lean_box(0); x_134 = x_153; -x_135 = x_145; -x_136 = x_146; -x_137 = x_151; -x_138 = x_155; +x_135 = x_146; +x_136 = x_155; +x_137 = x_145; +x_138 = x_151; x_139 = x_163; goto block_142; } @@ -48419,12 +48419,12 @@ if (x_176 == 0) { lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; x_177 = lean_ctor_get(x_175, 0); -x_178 = l_Lean_PersistentArray_append___redArg(x_165, x_177); +x_178 = l_Lean_PersistentArray_append___redArg(x_169, x_177); lean_dec_ref(x_177); lean_ctor_set(x_175, 0, x_178); x_179 = lean_st_ref_set(x_11, x_173); lean_dec(x_11); -x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_166); +x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_180; } else @@ -48434,7 +48434,7 @@ x_181 = lean_ctor_get_uint64(x_175, sizeof(void*)*1); x_182 = lean_ctor_get(x_175, 0); lean_inc(x_182); lean_dec(x_175); -x_183 = l_Lean_PersistentArray_append___redArg(x_165, x_182); +x_183 = l_Lean_PersistentArray_append___redArg(x_169, x_182); lean_dec_ref(x_182); x_184 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_184, 0, x_183); @@ -48442,7 +48442,7 @@ lean_ctor_set_uint64(x_184, sizeof(void*)*1, x_181); lean_ctor_set(x_173, 4, x_184); x_185 = lean_st_ref_set(x_11, x_173); lean_dec(x_11); -x_186 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_166); +x_186 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_186; } } @@ -48478,7 +48478,7 @@ if (lean_is_exclusive(x_187)) { lean_dec_ref(x_187); x_198 = lean_box(0); } -x_199 = l_Lean_PersistentArray_append___redArg(x_165, x_197); +x_199 = l_Lean_PersistentArray_append___redArg(x_169, x_197); lean_dec_ref(x_197); if (lean_is_scalar(x_198)) { x_200 = lean_alloc_ctor(0, 1, 8); @@ -48499,17 +48499,17 @@ lean_ctor_set(x_201, 7, x_194); lean_ctor_set(x_201, 8, x_195); x_202 = lean_st_ref_set(x_11, x_201); lean_dec(x_11); -x_203 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_166); +x_203 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__7___redArg(x_170); return x_203; } } else { x_81 = x_165; -x_82 = x_166; -x_83 = lean_box(0); -x_84 = x_168; -x_85 = x_169; +x_82 = lean_box(0); +x_83 = x_166; +x_84 = x_169; +x_85 = x_168; x_86 = x_170; goto block_90; } @@ -48517,10 +48517,10 @@ goto block_90; else { x_81 = x_165; -x_82 = x_166; -x_83 = lean_box(0); -x_84 = x_168; -x_85 = x_169; +x_82 = lean_box(0); +x_83 = x_166; +x_84 = x_169; +x_85 = x_168; x_86 = x_170; goto block_90; } @@ -48528,13 +48528,13 @@ goto block_90; block_214: { double x_212; uint8_t x_213; -x_212 = lean_float_sub(x_209, x_210); +x_212 = lean_float_sub(x_207, x_205); x_213 = lean_float_decLt(x_211, x_212); x_165 = x_205; -x_166 = x_206; +x_166 = x_207; x_167 = lean_box(0); -x_168 = x_208; -x_169 = x_209; +x_168 = x_209; +x_169 = x_208; x_170 = x_210; x_171 = x_213; goto block_204; @@ -48543,18 +48543,18 @@ goto block_204; { lean_object* x_220; double x_221; double x_222; lean_object* x_223; uint8_t x_224; x_220 = lean_io_get_num_heartbeats(); -x_221 = lean_float_of_nat(x_217); +x_221 = lean_float_of_nat(x_216); x_222 = lean_float_of_nat(x_220); x_223 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__3; x_224 = l_Lean_Option_get___at___00Lean_Elab_addMacroStack___at___00Lean_throwError___at___00Lean_Elab_Term_throwErrorIfErrors_spec__0_spec__1_spec__2(x_13, x_223); if (x_224 == 0) { -x_165 = x_216; -x_166 = x_218; +x_165 = x_221; +x_166 = x_222; x_167 = lean_box(0); x_168 = x_224; -x_169 = x_222; -x_170 = x_221; +x_169 = x_217; +x_170 = x_218; x_171 = x_224; goto block_204; } @@ -48568,12 +48568,12 @@ x_226 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_El x_227 = lean_float_of_nat(x_226); x_228 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__5; x_229 = lean_float_div(x_227, x_228); -x_205 = x_216; -x_206 = x_218; -x_207 = lean_box(0); -x_208 = x_224; -x_209 = x_222; -x_210 = x_221; +x_205 = x_221; +x_206 = lean_box(0); +x_207 = x_222; +x_208 = x_217; +x_209 = x_224; +x_210 = x_218; x_211 = x_229; goto block_214; } @@ -48583,12 +48583,12 @@ lean_object* x_230; lean_object* x_231; double x_232; x_230 = l_Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3___redArg___closed__4; x_231 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Elab_Term_TermElabM_0__Lean_Elab_Term_applyAttributesCore_spec__3_spec__8(x_13, x_230); x_232 = lean_float_of_nat(x_231); -x_205 = x_216; -x_206 = x_218; -x_207 = lean_box(0); -x_208 = x_224; -x_209 = x_222; -x_210 = x_221; +x_205 = x_221; +x_206 = lean_box(0); +x_207 = x_222; +x_208 = x_217; +x_209 = x_224; +x_210 = x_218; x_211 = x_232; goto block_214; } @@ -48621,8 +48621,8 @@ x_240 = !lean_is_exclusive(x_239); if (x_240 == 0) { lean_ctor_set_tag(x_239, 1); -x_143 = x_238; -x_144 = x_237; +x_143 = x_237; +x_144 = x_238; x_145 = x_235; x_146 = x_239; x_147 = lean_box(0); @@ -48636,8 +48636,8 @@ lean_inc(x_241); lean_dec(x_239); x_242 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_242, 0, x_241); -x_143 = x_238; -x_144 = x_237; +x_143 = x_237; +x_144 = x_238; x_145 = x_235; x_146 = x_242; x_147 = lean_box(0); @@ -48651,8 +48651,8 @@ x_243 = !lean_is_exclusive(x_239); if (x_243 == 0) { lean_ctor_set_tag(x_239, 0); -x_143 = x_238; -x_144 = x_237; +x_143 = x_237; +x_144 = x_238; x_145 = x_235; x_146 = x_239; x_147 = lean_box(0); @@ -48666,8 +48666,8 @@ lean_inc(x_244); lean_dec(x_239); x_245 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_245, 0, x_244); -x_143 = x_238; -x_144 = x_237; +x_143 = x_237; +x_144 = x_238; x_145 = x_235; x_146 = x_245; x_147 = lean_box(0); @@ -48694,8 +48694,8 @@ if (x_248 == 0) { lean_ctor_set_tag(x_247, 1); x_215 = x_237; -x_216 = x_235; -x_217 = x_246; +x_216 = x_246; +x_217 = x_235; x_218 = x_247; x_219 = lean_box(0); goto block_233; @@ -48709,8 +48709,8 @@ lean_dec(x_247); x_250 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_250, 0, x_249); x_215 = x_237; -x_216 = x_235; -x_217 = x_246; +x_216 = x_246; +x_217 = x_235; x_218 = x_250; x_219 = lean_box(0); goto block_233; @@ -48724,8 +48724,8 @@ if (x_251 == 0) { lean_ctor_set_tag(x_247, 0); x_215 = x_237; -x_216 = x_235; -x_217 = x_246; +x_216 = x_246; +x_217 = x_235; x_218 = x_247; x_219 = lean_box(0); goto block_233; @@ -48739,8 +48739,8 @@ lean_dec(x_247); x_253 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_253, 0, x_252); x_215 = x_237; -x_216 = x_235; -x_217 = x_246; +x_216 = x_246; +x_217 = x_235; x_218 = x_253; x_219 = lean_box(0); goto block_233; diff --git a/stage0/stdlib/Lean/Level.c b/stage0/stdlib/Lean/Level.c index 28ef4dfa9011..0a790df14b4f 100644 --- a/stage0/stdlib/Lean/Level.c +++ b/stage0/stdlib/Lean/Level.c @@ -8229,9 +8229,9 @@ goto block_52; block_44: { lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_nat_add(x_39, x_40); +x_41 = lean_nat_add(x_38, x_40); lean_dec(x_40); -lean_dec(x_39); +lean_dec(x_38); if (lean_is_scalar(x_35)) { x_42 = lean_alloc_ctor(0, 5, 0); } else { @@ -8250,7 +8250,7 @@ if (lean_is_scalar(x_25)) { lean_ctor_set(x_43, 0, x_37); lean_ctor_set(x_43, 1, x_28); lean_ctor_set(x_43, 2, x_29); -lean_ctor_set(x_43, 3, x_38); +lean_ctor_set(x_43, 3, x_39); lean_ctor_set(x_43, 4, x_42); return x_43; } @@ -8276,8 +8276,8 @@ if (lean_obj_tag(x_31) == 0) lean_object* x_50; x_50 = lean_ctor_get(x_31, 0); lean_inc(x_50); -x_38 = x_48; -x_39 = x_49; +x_38 = x_49; +x_39 = x_48; x_40 = x_50; goto block_44; } @@ -8285,8 +8285,8 @@ else { lean_object* x_51; x_51 = lean_unsigned_to_nat(0u); -x_38 = x_48; -x_39 = x_49; +x_38 = x_49; +x_39 = x_48; x_40 = x_51; goto block_44; } diff --git a/stage0/stdlib/Lean/Meta/ArgsPacker.c b/stage0/stdlib/Lean/Meta/ArgsPacker.c index a4e3bda2a148..171b02c53b76 100644 --- a/stage0/stdlib/Lean/Meta/ArgsPacker.c +++ b/stage0/stdlib/Lean/Meta/ArgsPacker.c @@ -8713,15 +8713,15 @@ goto block_49; { lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_inc(x_3); -x_22 = l_List_get_x21Internal___redArg(x_13, x_15, x_3); -lean_dec(x_15); +x_22 = l_List_get_x21Internal___redArg(x_13, x_16, x_3); +lean_dec(x_16); x_23 = l_Lean_Expr_bindingName_x21(x_12); lean_dec(x_12); lean_inc(x_20); lean_inc_ref(x_19); lean_inc(x_18); lean_inc_ref(x_17); -x_24 = l_Lean_Meta_withLocalDeclD___at___00Lean_Meta_ArgsPacker_Unary_uncurryType_spec__1___redArg(x_23, x_22, x_16, x_17, x_18, x_19, x_20); +x_24 = l_Lean_Meta_withLocalDeclD___at___00Lean_Meta_ArgsPacker_Unary_uncurryType_spec__1___redArg(x_23, x_22, x_15, x_17, x_18, x_19, x_20); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; lean_object* x_27; @@ -8797,8 +8797,8 @@ return x_45; } else { -x_15 = x_37; -x_16 = x_38; +x_15 = x_38; +x_16 = x_37; x_17 = x_30; x_18 = x_31; x_19 = x_32; diff --git a/stage0/stdlib/Lean/Meta/IndPredBelow.c b/stage0/stdlib/Lean/Meta/IndPredBelow.c index 7e5d31472e3a..99ec1af68d94 100644 --- a/stage0/stdlib/Lean/Meta/IndPredBelow.c +++ b/stage0/stdlib/Lean/Meta/IndPredBelow.c @@ -5723,7 +5723,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg(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) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_28; lean_object* x_29; double x_30; uint8_t x_31; double x_32; lean_object* x_33; lean_object* x_34; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; double x_43; double x_44; 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; double x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; double x_68; lean_object* x_69; lean_object* x_70; double x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; double x_79; lean_object* x_80; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; double x_90; uint8_t x_91; double x_92; uint8_t x_93; lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; double x_131; double x_132; double x_133; lean_object* x_137; uint8_t x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; double x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; double x_163; lean_object* x_164; uint8_t x_165; double x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; double x_203; lean_object* x_204; double x_205; lean_object* x_209; uint8_t x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; +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; double x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; double x_32; lean_object* x_33; lean_object* x_34; lean_object* x_39; lean_object* x_40; double x_41; lean_object* x_42; uint8_t x_43; double x_44; 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_64; lean_object* x_65; double x_66; double x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_75; lean_object* x_76; lean_object* x_77; double x_78; double x_79; uint8_t x_80; lean_object* x_85; lean_object* x_86; lean_object* x_87; double x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; double x_92; uint8_t x_93; lean_object* x_127; lean_object* x_128; double x_129; lean_object* x_130; uint8_t x_131; double x_132; double x_133; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_159; lean_object* x_160; lean_object* x_161; double x_162; double x_163; uint8_t x_164; uint8_t x_165; lean_object* x_199; lean_object* x_200; lean_object* x_201; double x_202; double x_203; uint8_t x_204; double x_205; uint8_t x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; x_11 = lean_ctor_get(x_8, 2); x_12 = lean_ctor_get(x_8, 5); lean_inc(x_1); @@ -5805,8 +5805,8 @@ lean_ctor_set(x_36, 1, x_5); lean_ctor_set_float(x_36, sizeof(void*)*2, x_35); lean_ctor_set_float(x_36, sizeof(void*)*2 + 8, x_35); lean_ctor_set_uint8(x_36, sizeof(void*)*2 + 16, x_4); -x_13 = x_28; -x_14 = x_29; +x_13 = x_29; +x_14 = x_30; x_15 = x_33; x_16 = x_36; x_17 = x_6; @@ -5822,11 +5822,11 @@ lean_object* x_37; x_37 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_37, 0, x_1); lean_ctor_set(x_37, 1, x_5); -lean_ctor_set_float(x_37, sizeof(void*)*2, x_30); -lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_32); +lean_ctor_set_float(x_37, sizeof(void*)*2, x_32); +lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_28); lean_ctor_set_uint8(x_37, sizeof(void*)*2 + 16, x_4); -x_13 = x_28; -x_14 = x_29; +x_13 = x_29; +x_14 = x_30; x_15 = x_33; x_16 = x_37; x_17 = x_6; @@ -5844,18 +5844,18 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_41); -x_45 = lean_apply_6(x_2, x_41, x_6, x_7, x_8, x_9, lean_box(0)); +lean_inc_ref(x_42); +x_45 = lean_apply_6(x_2, x_42, x_6, x_7, x_8, x_9, lean_box(0)); if (lean_obj_tag(x_45) == 0) { lean_object* x_46; x_46 = lean_ctor_get(x_45, 0); lean_inc(x_46); lean_dec_ref(x_45); -x_28 = x_40; -x_29 = x_41; -x_30 = x_43; -x_31 = x_42; +x_28 = x_41; +x_29 = x_40; +x_30 = x_42; +x_31 = x_43; x_32 = x_44; x_33 = x_46; x_34 = lean_box(0); @@ -5866,10 +5866,10 @@ else lean_object* x_47; lean_dec_ref(x_45); x_47 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__2; -x_28 = x_40; -x_29 = x_41; -x_30 = x_43; -x_31 = x_42; +x_28 = x_41; +x_29 = x_40; +x_30 = x_42; +x_31 = x_43; x_32 = x_44; x_33 = x_47; x_34 = lean_box(0); @@ -5913,7 +5913,7 @@ return x_62; } block_74: { -if (x_67 == 0) +if (x_68 == 0) { double x_71; lean_object* x_72; x_71 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__0; @@ -5923,8 +5923,8 @@ lean_ctor_set(x_72, 1, x_5); lean_ctor_set_float(x_72, sizeof(void*)*2, x_71); lean_ctor_set_float(x_72, sizeof(void*)*2 + 8, x_71); lean_ctor_set_uint8(x_72, sizeof(void*)*2 + 16, x_4); -x_49 = x_65; -x_50 = x_66; +x_49 = x_64; +x_50 = x_65; x_51 = x_69; x_52 = x_72; x_53 = x_6; @@ -5940,11 +5940,11 @@ lean_object* x_73; x_73 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_73, 0, x_1); lean_ctor_set(x_73, 1, x_5); -lean_ctor_set_float(x_73, sizeof(void*)*2, x_68); -lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_64); +lean_ctor_set_float(x_73, sizeof(void*)*2, x_67); +lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_66); lean_ctor_set_uint8(x_73, sizeof(void*)*2 + 16, x_4); -x_49 = x_65; -x_50 = x_66; +x_49 = x_64; +x_50 = x_65; x_51 = x_69; x_52 = x_73; x_53 = x_6; @@ -5971,10 +5971,10 @@ x_82 = lean_ctor_get(x_81, 0); lean_inc(x_82); lean_dec_ref(x_81); x_64 = x_75; -x_65 = x_76; -x_66 = x_77; -x_67 = x_78; -x_68 = x_79; +x_65 = x_77; +x_66 = x_78; +x_67 = x_79; +x_68 = x_80; x_69 = x_82; x_70 = lean_box(0); goto block_74; @@ -5985,10 +5985,10 @@ lean_object* x_83; lean_dec_ref(x_81); x_83 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__2; x_64 = x_75; -x_65 = x_76; -x_66 = x_77; -x_67 = x_78; -x_68 = x_79; +x_65 = x_77; +x_66 = x_78; +x_67 = x_79; +x_68 = x_80; x_69 = x_83; x_70 = lean_box(0); goto block_74; @@ -6022,12 +6022,12 @@ if (x_98 == 0) { lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; x_99 = lean_ctor_get(x_97, 0); -x_100 = l_Lean_PersistentArray_append___redArg(x_87, x_99); +x_100 = l_Lean_PersistentArray_append___redArg(x_89, x_99); lean_dec_ref(x_99); lean_ctor_set(x_97, 0, x_100); x_101 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_89); +x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_90); return x_102; } else @@ -6037,7 +6037,7 @@ x_103 = lean_ctor_get_uint64(x_97, sizeof(void*)*1); x_104 = lean_ctor_get(x_97, 0); lean_inc(x_104); lean_dec(x_97); -x_105 = l_Lean_PersistentArray_append___redArg(x_87, x_104); +x_105 = l_Lean_PersistentArray_append___redArg(x_89, x_104); lean_dec_ref(x_104); x_106 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_106, 0, x_105); @@ -6045,7 +6045,7 @@ lean_ctor_set_uint64(x_106, sizeof(void*)*1, x_103); lean_ctor_set(x_95, 4, x_106); x_107 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_89); +x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_90); return x_108; } } @@ -6081,7 +6081,7 @@ if (lean_is_exclusive(x_109)) { lean_dec_ref(x_109); x_120 = lean_box(0); } -x_121 = l_Lean_PersistentArray_append___redArg(x_87, x_119); +x_121 = l_Lean_PersistentArray_append___redArg(x_89, x_119); lean_dec_ref(x_119); if (lean_is_scalar(x_120)) { x_122 = lean_alloc_ctor(0, 1, 8); @@ -6102,17 +6102,17 @@ lean_ctor_set(x_123, 7, x_116); lean_ctor_set(x_123, 8, x_117); x_124 = lean_st_ref_set(x_9, x_123); lean_dec(x_9); -x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_89); +x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__14___redArg(x_90); return x_125; } } else { x_39 = lean_box(0); -x_40 = x_87; -x_41 = x_89; -x_42 = x_91; -x_43 = x_90; +x_40 = x_89; +x_41 = x_88; +x_42 = x_90; +x_43 = x_91; x_44 = x_92; goto block_48; } @@ -6120,10 +6120,10 @@ goto block_48; else { x_39 = lean_box(0); -x_40 = x_87; -x_41 = x_89; -x_42 = x_91; -x_43 = x_90; +x_40 = x_89; +x_41 = x_88; +x_42 = x_90; +x_43 = x_91; x_44 = x_92; goto block_48; } @@ -6131,13 +6131,13 @@ goto block_48; block_136: { double x_134; uint8_t x_135; -x_134 = lean_float_sub(x_132, x_131); +x_134 = lean_float_sub(x_129, x_132); x_135 = lean_float_decLt(x_133, x_134); -x_87 = x_128; -x_88 = lean_box(0); -x_89 = x_129; -x_90 = x_131; -x_91 = x_130; +x_87 = lean_box(0); +x_88 = x_129; +x_89 = x_128; +x_90 = x_130; +x_91 = x_131; x_92 = x_132; x_93 = x_135; goto block_126; @@ -6155,18 +6155,18 @@ x_148 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___r x_149 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__12(x_11, x_148); if (x_149 == 0) { -x_87 = x_137; -x_88 = lean_box(0); -x_89 = x_140; -x_90 = x_145; +x_87 = lean_box(0); +x_88 = x_147; +x_89 = x_138; +x_90 = x_140; x_91 = x_149; -x_92 = x_147; +x_92 = x_145; x_93 = x_149; goto block_126; } else { -if (x_138 == 0) +if (x_137 == 0) { lean_object* x_150; lean_object* x_151; double x_152; double x_153; double x_154; x_150 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; @@ -6175,11 +6175,11 @@ x_152 = lean_float_of_nat(x_151); x_153 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__6; x_154 = lean_float_div(x_152, x_153); x_127 = lean_box(0); -x_128 = x_137; -x_129 = x_140; -x_130 = x_149; -x_131 = x_145; -x_132 = x_147; +x_128 = x_138; +x_129 = x_147; +x_130 = x_140; +x_131 = x_149; +x_132 = x_145; x_133 = x_154; goto block_136; } @@ -6190,11 +6190,11 @@ x_155 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___r x_156 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__15(x_11, x_155); x_157 = lean_float_of_nat(x_156); x_127 = lean_box(0); -x_128 = x_137; -x_129 = x_140; -x_130 = x_149; -x_131 = x_145; -x_132 = x_147; +x_128 = x_138; +x_129 = x_147; +x_130 = x_140; +x_131 = x_149; +x_132 = x_145; x_133 = x_157; goto block_136; } @@ -6228,7 +6228,7 @@ if (x_170 == 0) { lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; x_171 = lean_ctor_get(x_169, 0); -x_172 = l_Lean_PersistentArray_append___redArg(x_160, x_171); +x_172 = l_Lean_PersistentArray_append___redArg(x_159, x_171); lean_dec_ref(x_171); lean_ctor_set(x_169, 0, x_172); x_173 = lean_st_ref_set(x_9, x_167); @@ -6243,7 +6243,7 @@ x_175 = lean_ctor_get_uint64(x_169, sizeof(void*)*1); x_176 = lean_ctor_get(x_169, 0); lean_inc(x_176); lean_dec(x_169); -x_177 = l_Lean_PersistentArray_append___redArg(x_160, x_176); +x_177 = l_Lean_PersistentArray_append___redArg(x_159, x_176); lean_dec_ref(x_176); x_178 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_178, 0, x_177); @@ -6287,7 +6287,7 @@ if (lean_is_exclusive(x_181)) { lean_dec_ref(x_181); x_192 = lean_box(0); } -x_193 = l_Lean_PersistentArray_append___redArg(x_160, x_191); +x_193 = l_Lean_PersistentArray_append___redArg(x_159, x_191); lean_dec_ref(x_191); if (lean_is_scalar(x_192)) { x_194 = lean_alloc_ctor(0, 1, 8); @@ -6315,36 +6315,36 @@ return x_197; else { x_75 = x_159; -x_76 = x_160; +x_76 = lean_box(0); x_77 = x_161; x_78 = x_162; x_79 = x_163; -x_80 = lean_box(0); +x_80 = x_164; goto block_84; } } else { x_75 = x_159; -x_76 = x_160; +x_76 = lean_box(0); x_77 = x_161; x_78 = x_162; x_79 = x_163; -x_80 = lean_box(0); +x_80 = x_164; goto block_84; } } block_208: { double x_206; uint8_t x_207; -x_206 = lean_float_sub(x_199, x_203); +x_206 = lean_float_sub(x_202, x_203); x_207 = lean_float_decLt(x_205, x_206); x_159 = x_199; -x_160 = x_200; +x_160 = lean_box(0); x_161 = x_201; x_162 = x_202; x_163 = x_203; -x_164 = lean_box(0); +x_164 = x_204; x_165 = x_207; goto block_198; } @@ -6358,18 +6358,18 @@ x_217 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___r x_218 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__12(x_11, x_217); if (x_218 == 0) { -x_159 = x_216; -x_160 = x_209; +x_159 = x_210; +x_160 = lean_box(0); x_161 = x_212; -x_162 = x_218; +x_162 = x_216; x_163 = x_215; -x_164 = lean_box(0); +x_164 = x_218; x_165 = x_218; goto block_198; } else { -if (x_210 == 0) +if (x_209 == 0) { lean_object* x_219; lean_object* x_220; double x_221; double x_222; double x_223; x_219 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; @@ -6377,12 +6377,12 @@ x_220 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPred x_221 = lean_float_of_nat(x_220); x_222 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__6; x_223 = lean_float_div(x_221, x_222); -x_199 = x_216; -x_200 = x_209; +x_199 = x_210; +x_200 = lean_box(0); x_201 = x_212; -x_202 = x_218; +x_202 = x_216; x_203 = x_215; -x_204 = lean_box(0); +x_204 = x_218; x_205 = x_223; goto block_208; } @@ -6392,12 +6392,12 @@ lean_object* x_224; lean_object* x_225; double x_226; x_224 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; x_225 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__15(x_11, x_224); x_226 = lean_float_of_nat(x_225); -x_199 = x_216; -x_200 = x_209; +x_199 = x_210; +x_200 = lean_box(0); x_201 = x_212; -x_202 = x_218; +x_202 = x_216; x_203 = x_215; -x_204 = lean_box(0); +x_204 = x_218; x_205 = x_226; goto block_208; } @@ -6428,8 +6428,8 @@ x_234 = !lean_is_exclusive(x_233); if (x_234 == 0) { lean_ctor_set_tag(x_233, 1); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_233; x_141 = lean_box(0); @@ -6443,8 +6443,8 @@ lean_inc(x_235); lean_dec(x_233); x_236 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_236, 0, x_235); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_236; x_141 = lean_box(0); @@ -6458,8 +6458,8 @@ x_237 = !lean_is_exclusive(x_233); if (x_237 == 0) { lean_ctor_set_tag(x_233, 0); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_233; x_141 = lean_box(0); @@ -6473,8 +6473,8 @@ lean_inc(x_238); lean_dec(x_233); x_239 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_239, 0, x_238); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_239; x_141 = lean_box(0); @@ -6498,8 +6498,8 @@ x_242 = !lean_is_exclusive(x_241); if (x_242 == 0) { lean_ctor_set_tag(x_241, 1); -x_209 = x_229; -x_210 = x_231; +x_209 = x_231; +x_210 = x_229; x_211 = x_240; x_212 = x_241; x_213 = lean_box(0); @@ -6513,8 +6513,8 @@ lean_inc(x_243); lean_dec(x_241); x_244 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_244, 0, x_243); -x_209 = x_229; -x_210 = x_231; +x_209 = x_231; +x_210 = x_229; x_211 = x_240; x_212 = x_244; x_213 = lean_box(0); @@ -6528,8 +6528,8 @@ x_245 = !lean_is_exclusive(x_241); if (x_245 == 0) { lean_ctor_set_tag(x_241, 0); -x_209 = x_229; -x_210 = x_231; +x_209 = x_231; +x_210 = x_229; x_211 = x_240; x_212 = x_241; x_213 = lean_box(0); @@ -6543,8 +6543,8 @@ lean_inc(x_246); lean_dec(x_241); x_247 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_247, 0, x_246); -x_209 = x_229; -x_210 = x_231; +x_209 = x_231; +x_210 = x_229; x_211 = x_240; x_212 = x_247; x_213 = lean_box(0); @@ -11202,7 +11202,7 @@ return x_34; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8___redArg(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_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_30; lean_object* x_31; lean_object* x_32; double x_33; double x_34; lean_object* x_35; lean_object* x_36; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; double x_45; double x_46; 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_67; uint8_t x_68; double x_69; lean_object* x_70; double x_71; lean_object* x_72; lean_object* x_73; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; double x_82; double x_83; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; double x_94; double x_95; uint8_t x_96; lean_object* x_130; uint8_t x_131; lean_object* x_132; lean_object* x_133; double x_134; double x_135; double x_136; uint8_t x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_162; uint8_t x_163; double x_164; lean_object* x_165; lean_object* x_166; double x_167; uint8_t x_168; lean_object* x_202; uint8_t x_203; lean_object* x_204; lean_object* x_205; double x_206; double x_207; double x_208; uint8_t x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; uint8_t x_252; +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_30; uint8_t x_31; double x_32; double x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_41; uint8_t x_42; lean_object* x_43; double x_44; double x_45; lean_object* x_46; 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_67; lean_object* x_68; double x_69; double x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; lean_object* x_78; lean_object* x_79; double x_80; lean_object* x_81; double x_82; uint8_t x_83; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; double x_92; lean_object* x_93; double x_94; lean_object* x_95; uint8_t x_96; lean_object* x_130; uint8_t x_131; lean_object* x_132; double x_133; double x_134; lean_object* x_135; double x_136; lean_object* x_140; uint8_t x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_162; lean_object* x_163; double x_164; lean_object* x_165; double x_166; uint8_t x_167; uint8_t x_168; lean_object* x_202; lean_object* x_203; double x_204; lean_object* x_205; double x_206; uint8_t x_207; double x_208; lean_object* x_212; uint8_t x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; uint8_t x_252; x_12 = lean_ctor_get(x_9, 2); x_13 = lean_ctor_get(x_9, 5); lean_inc(x_1); @@ -11241,7 +11241,7 @@ goto block_251; { lean_object* x_24; lean_dec(x_18); -x_24 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__11___redArg(x_15, x_17, x_13, x_16, x_19, x_20, x_21, x_22); +x_24 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__11___redArg(x_14, x_17, x_13, x_16, x_19, x_20, x_21, x_22); lean_dec(x_22); lean_dec(x_20); lean_dec_ref(x_19); @@ -11249,13 +11249,13 @@ if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_dec_ref(x_24); -x_25 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_14); +x_25 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_15); return x_25; } else { uint8_t x_26; -lean_dec_ref(x_14); +lean_dec_ref(x_15); x_26 = !lean_is_exclusive(x_24); if (x_26 == 0) { @@ -11275,7 +11275,7 @@ return x_28; } block_40: { -if (x_30 == 0) +if (x_31 == 0) { double x_37; lean_object* x_38; x_37 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__0; @@ -11285,8 +11285,8 @@ lean_ctor_set(x_38, 1, x_5); lean_ctor_set_float(x_38, sizeof(void*)*2, x_37); lean_ctor_set_float(x_38, sizeof(void*)*2 + 8, x_37); lean_ctor_set_uint8(x_38, sizeof(void*)*2 + 16, x_4); -x_14 = x_32; -x_15 = x_31; +x_14 = x_30; +x_15 = x_34; x_16 = x_35; x_17 = x_38; x_18 = x_6; @@ -11303,11 +11303,11 @@ lean_object* x_39; x_39 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_39, 0, x_1); lean_ctor_set(x_39, 1, x_5); -lean_ctor_set_float(x_39, sizeof(void*)*2, x_34); -lean_ctor_set_float(x_39, sizeof(void*)*2 + 8, x_33); +lean_ctor_set_float(x_39, sizeof(void*)*2, x_33); +lean_ctor_set_float(x_39, sizeof(void*)*2 + 8, x_32); lean_ctor_set_uint8(x_39, sizeof(void*)*2 + 16, x_4); -x_14 = x_32; -x_15 = x_31; +x_14 = x_30; +x_15 = x_34; x_16 = x_35; x_17 = x_39; x_18 = x_6; @@ -11327,17 +11327,17 @@ lean_inc_ref(x_9); lean_inc(x_8); lean_inc_ref(x_7); lean_inc(x_6); -lean_inc_ref(x_43); -x_47 = lean_apply_7(x_2, x_43, x_6, x_7, x_8, x_9, x_10, lean_box(0)); +lean_inc_ref(x_46); +x_47 = lean_apply_7(x_2, x_46, x_6, x_7, x_8, x_9, x_10, lean_box(0)); if (lean_obj_tag(x_47) == 0) { lean_object* x_48; x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); lean_dec_ref(x_47); -x_30 = x_42; -x_31 = x_44; -x_32 = x_43; +x_30 = x_41; +x_31 = x_42; +x_32 = x_44; x_33 = x_45; x_34 = x_46; x_35 = x_48; @@ -11349,9 +11349,9 @@ else lean_object* x_49; lean_dec_ref(x_47); x_49 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__2; -x_30 = x_42; -x_31 = x_44; -x_32 = x_43; +x_30 = x_41; +x_31 = x_42; +x_32 = x_44; x_33 = x_45; x_34 = x_46; x_35 = x_49; @@ -11363,7 +11363,7 @@ goto block_40; { lean_object* x_61; lean_dec(x_55); -x_61 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__11___redArg(x_53, x_54, x_13, x_51, x_56, x_57, x_58, x_59); +x_61 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__11___redArg(x_51, x_54, x_13, x_53, x_56, x_57, x_58, x_59); lean_dec(x_59); lean_dec(x_57); lean_dec_ref(x_56); @@ -11397,7 +11397,7 @@ return x_65; } block_77: { -if (x_68 == 0) +if (x_71 == 0) { double x_74; lean_object* x_75; x_74 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__0; @@ -11407,9 +11407,9 @@ lean_ctor_set(x_75, 1, x_5); lean_ctor_set_float(x_75, sizeof(void*)*2, x_74); lean_ctor_set_float(x_75, sizeof(void*)*2 + 8, x_74); lean_ctor_set_uint8(x_75, sizeof(void*)*2 + 16, x_4); -x_51 = x_72; -x_52 = x_67; -x_53 = x_70; +x_51 = x_67; +x_52 = x_68; +x_53 = x_72; x_54 = x_75; x_55 = x_6; x_56 = x_7; @@ -11426,11 +11426,11 @@ x_76 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_76, 0, x_1); lean_ctor_set(x_76, 1, x_5); lean_ctor_set_float(x_76, sizeof(void*)*2, x_69); -lean_ctor_set_float(x_76, sizeof(void*)*2 + 8, x_71); +lean_ctor_set_float(x_76, sizeof(void*)*2 + 8, x_70); lean_ctor_set_uint8(x_76, sizeof(void*)*2 + 16, x_4); -x_51 = x_72; -x_52 = x_67; -x_53 = x_70; +x_51 = x_67; +x_52 = x_68; +x_53 = x_72; x_54 = x_76; x_55 = x_6; x_56 = x_7; @@ -11449,8 +11449,8 @@ lean_inc_ref(x_9); lean_inc(x_8); lean_inc_ref(x_7); lean_inc(x_6); -lean_inc_ref(x_78); -x_84 = lean_apply_7(x_2, x_78, x_6, x_7, x_8, x_9, x_10, lean_box(0)); +lean_inc_ref(x_79); +x_84 = lean_apply_7(x_2, x_79, x_6, x_7, x_8, x_9, x_10, lean_box(0)); if (lean_obj_tag(x_84) == 0) { lean_object* x_85; @@ -11459,8 +11459,8 @@ lean_inc(x_85); lean_dec_ref(x_84); x_67 = x_78; x_68 = x_79; -x_69 = x_82; -x_70 = x_81; +x_69 = x_80; +x_70 = x_82; x_71 = x_83; x_72 = x_85; x_73 = lean_box(0); @@ -11473,8 +11473,8 @@ lean_dec_ref(x_84); x_86 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__2; x_67 = x_78; x_68 = x_79; -x_69 = x_82; -x_70 = x_81; +x_69 = x_80; +x_70 = x_82; x_71 = x_83; x_72 = x_86; x_73 = lean_box(0); @@ -11510,12 +11510,12 @@ if (x_101 == 0) { lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; x_102 = lean_ctor_get(x_100, 0); -x_103 = l_Lean_PersistentArray_append___redArg(x_93, x_102); +x_103 = l_Lean_PersistentArray_append___redArg(x_90, x_102); lean_dec_ref(x_102); lean_ctor_set(x_100, 0, x_103); x_104 = lean_st_ref_set(x_10, x_98); lean_dec(x_10); -x_105 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_92); +x_105 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_95); return x_105; } else @@ -11525,7 +11525,7 @@ x_106 = lean_ctor_get_uint64(x_100, sizeof(void*)*1); x_107 = lean_ctor_get(x_100, 0); lean_inc(x_107); lean_dec(x_100); -x_108 = l_Lean_PersistentArray_append___redArg(x_93, x_107); +x_108 = l_Lean_PersistentArray_append___redArg(x_90, x_107); lean_dec_ref(x_107); x_109 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_109, 0, x_108); @@ -11533,7 +11533,7 @@ lean_ctor_set_uint64(x_109, sizeof(void*)*1, x_106); lean_ctor_set(x_98, 4, x_109); x_110 = lean_st_ref_set(x_10, x_98); lean_dec(x_10); -x_111 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_92); +x_111 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_95); return x_111; } } @@ -11569,7 +11569,7 @@ if (lean_is_exclusive(x_112)) { lean_dec_ref(x_112); x_123 = lean_box(0); } -x_124 = l_Lean_PersistentArray_append___redArg(x_93, x_122); +x_124 = l_Lean_PersistentArray_append___redArg(x_90, x_122); lean_dec_ref(x_122); if (lean_is_scalar(x_123)) { x_125 = lean_alloc_ctor(0, 1, 8); @@ -11590,16 +11590,16 @@ lean_ctor_set(x_126, 7, x_119); lean_ctor_set(x_126, 8, x_120); x_127 = lean_st_ref_set(x_10, x_126); lean_dec(x_10); -x_128 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_92); +x_128 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_95); return x_128; } } else { -x_41 = lean_box(0); +x_41 = x_90; x_42 = x_91; -x_43 = x_92; -x_44 = x_93; +x_43 = lean_box(0); +x_44 = x_92; x_45 = x_94; x_46 = x_95; goto block_50; @@ -11607,10 +11607,10 @@ goto block_50; } else { -x_41 = lean_box(0); +x_41 = x_90; x_42 = x_91; -x_43 = x_92; -x_44 = x_93; +x_43 = lean_box(0); +x_44 = x_92; x_45 = x_94; x_46 = x_95; goto block_50; @@ -11619,12 +11619,12 @@ goto block_50; block_139: { double x_137; uint8_t x_138; -x_137 = lean_float_sub(x_134, x_135); +x_137 = lean_float_sub(x_133, x_134); x_138 = lean_float_decLt(x_136, x_137); -x_90 = lean_box(0); +x_90 = x_130; x_91 = x_131; x_92 = x_133; -x_93 = x_132; +x_93 = lean_box(0); x_94 = x_134; x_95 = x_135; x_96 = x_138; @@ -11634,7 +11634,7 @@ goto block_129; { lean_object* x_145; double x_146; double x_147; double x_148; double x_149; double x_150; lean_object* x_151; uint8_t x_152; x_145 = lean_io_mono_nanos_now(); -x_146 = lean_float_of_nat(x_141); +x_146 = lean_float_of_nat(x_142); x_147 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__3; x_148 = lean_float_div(x_146, x_147); x_149 = lean_float_of_nat(x_145); @@ -11643,18 +11643,18 @@ x_151 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___r x_152 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__12(x_12, x_151); if (x_152 == 0) { -x_90 = lean_box(0); +x_90 = x_140; x_91 = x_152; -x_92 = x_143; -x_93 = x_142; -x_94 = x_150; -x_95 = x_148; +x_92 = x_150; +x_93 = lean_box(0); +x_94 = x_148; +x_95 = x_143; x_96 = x_152; goto block_129; } else { -if (x_140 == 0) +if (x_141 == 0) { lean_object* x_153; lean_object* x_154; double x_155; double x_156; double x_157; x_153 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; @@ -11662,12 +11662,12 @@ x_154 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPred x_155 = lean_float_of_nat(x_154); x_156 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__6; x_157 = lean_float_div(x_155, x_156); -x_130 = lean_box(0); +x_130 = x_140; x_131 = x_152; -x_132 = x_142; -x_133 = x_143; -x_134 = x_150; -x_135 = x_148; +x_132 = lean_box(0); +x_133 = x_150; +x_134 = x_148; +x_135 = x_143; x_136 = x_157; goto block_139; } @@ -11677,12 +11677,12 @@ lean_object* x_158; lean_object* x_159; double x_160; x_158 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; x_159 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__15(x_12, x_158); x_160 = lean_float_of_nat(x_159); -x_130 = lean_box(0); +x_130 = x_140; x_131 = x_152; -x_132 = x_142; -x_133 = x_143; -x_134 = x_150; -x_135 = x_148; +x_132 = lean_box(0); +x_133 = x_150; +x_134 = x_148; +x_135 = x_143; x_136 = x_160; goto block_139; } @@ -11717,12 +11717,12 @@ if (x_173 == 0) { lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; x_174 = lean_ctor_get(x_172, 0); -x_175 = l_Lean_PersistentArray_append___redArg(x_165, x_174); +x_175 = l_Lean_PersistentArray_append___redArg(x_162, x_174); lean_dec_ref(x_174); lean_ctor_set(x_172, 0, x_175); x_176 = lean_st_ref_set(x_10, x_170); lean_dec(x_10); -x_177 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_162); +x_177 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_163); return x_177; } else @@ -11732,7 +11732,7 @@ x_178 = lean_ctor_get_uint64(x_172, sizeof(void*)*1); x_179 = lean_ctor_get(x_172, 0); lean_inc(x_179); lean_dec(x_172); -x_180 = l_Lean_PersistentArray_append___redArg(x_165, x_179); +x_180 = l_Lean_PersistentArray_append___redArg(x_162, x_179); lean_dec_ref(x_179); x_181 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_181, 0, x_180); @@ -11740,7 +11740,7 @@ lean_ctor_set_uint64(x_181, sizeof(void*)*1, x_178); lean_ctor_set(x_170, 4, x_181); x_182 = lean_st_ref_set(x_10, x_170); lean_dec(x_10); -x_183 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_162); +x_183 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_163); return x_183; } } @@ -11776,7 +11776,7 @@ if (lean_is_exclusive(x_184)) { lean_dec_ref(x_184); x_195 = lean_box(0); } -x_196 = l_Lean_PersistentArray_append___redArg(x_165, x_194); +x_196 = l_Lean_PersistentArray_append___redArg(x_162, x_194); lean_dec_ref(x_194); if (lean_is_scalar(x_195)) { x_197 = lean_alloc_ctor(0, 1, 8); @@ -11797,7 +11797,7 @@ lean_ctor_set(x_198, 7, x_191); lean_ctor_set(x_198, 8, x_192); x_199 = lean_st_ref_set(x_10, x_198); lean_dec(x_10); -x_200 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_162); +x_200 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__8_spec__12___redArg(x_163); return x_200; } } @@ -11805,9 +11805,9 @@ else { x_78 = x_162; x_79 = x_163; -x_80 = lean_box(0); -x_81 = x_165; -x_82 = x_164; +x_80 = x_164; +x_81 = lean_box(0); +x_82 = x_166; x_83 = x_167; goto block_87; } @@ -11816,9 +11816,9 @@ else { x_78 = x_162; x_79 = x_163; -x_80 = lean_box(0); -x_81 = x_165; -x_82 = x_164; +x_80 = x_164; +x_81 = lean_box(0); +x_82 = x_166; x_83 = x_167; goto block_87; } @@ -11826,13 +11826,13 @@ goto block_87; block_211: { double x_209; uint8_t x_210; -x_209 = lean_float_sub(x_207, x_206); +x_209 = lean_float_sub(x_206, x_204); x_210 = lean_float_decLt(x_208, x_209); x_162 = x_202; x_163 = x_203; -x_164 = x_206; -x_165 = x_205; -x_166 = lean_box(0); +x_164 = x_204; +x_165 = lean_box(0); +x_166 = x_206; x_167 = x_207; x_168 = x_210; goto block_201; @@ -11841,24 +11841,24 @@ goto block_201; { lean_object* x_217; double x_218; double x_219; lean_object* x_220; uint8_t x_221; x_217 = lean_io_get_num_heartbeats(); -x_218 = lean_float_of_nat(x_213); +x_218 = lean_float_of_nat(x_214); x_219 = lean_float_of_nat(x_217); x_220 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__4; x_221 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__12(x_12, x_220); if (x_221 == 0) { -x_162 = x_215; -x_163 = x_221; +x_162 = x_212; +x_163 = x_215; x_164 = x_218; -x_165 = x_214; -x_166 = lean_box(0); -x_167 = x_219; +x_165 = lean_box(0); +x_166 = x_219; +x_167 = x_221; x_168 = x_221; goto block_201; } else { -if (x_212 == 0) +if (x_213 == 0) { lean_object* x_222; lean_object* x_223; double x_224; double x_225; double x_226; x_222 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; @@ -11866,12 +11866,12 @@ x_223 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPred x_224 = lean_float_of_nat(x_223); x_225 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__6; x_226 = lean_float_div(x_224, x_225); -x_202 = x_215; -x_203 = x_221; -x_204 = lean_box(0); -x_205 = x_214; -x_206 = x_218; -x_207 = x_219; +x_202 = x_212; +x_203 = x_215; +x_204 = x_218; +x_205 = lean_box(0); +x_206 = x_219; +x_207 = x_221; x_208 = x_226; goto block_211; } @@ -11881,12 +11881,12 @@ lean_object* x_227; lean_object* x_228; double x_229; x_227 = l_Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8___redArg___closed__5; x_228 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__15(x_12, x_227); x_229 = lean_float_of_nat(x_228); -x_202 = x_215; -x_203 = x_221; -x_204 = lean_box(0); -x_205 = x_214; -x_206 = x_218; -x_207 = x_219; +x_202 = x_212; +x_203 = x_215; +x_204 = x_218; +x_205 = lean_box(0); +x_206 = x_219; +x_207 = x_221; x_208 = x_229; goto block_211; } @@ -11918,9 +11918,9 @@ x_237 = !lean_is_exclusive(x_236); if (x_237 == 0) { lean_ctor_set_tag(x_236, 1); -x_140 = x_234; -x_141 = x_235; -x_142 = x_232; +x_140 = x_232; +x_141 = x_234; +x_142 = x_235; x_143 = x_236; x_144 = lean_box(0); goto block_161; @@ -11933,9 +11933,9 @@ lean_inc(x_238); lean_dec(x_236); x_239 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_239, 0, x_238); -x_140 = x_234; -x_141 = x_235; -x_142 = x_232; +x_140 = x_232; +x_141 = x_234; +x_142 = x_235; x_143 = x_239; x_144 = lean_box(0); goto block_161; @@ -11948,9 +11948,9 @@ x_240 = !lean_is_exclusive(x_236); if (x_240 == 0) { lean_ctor_set_tag(x_236, 0); -x_140 = x_234; -x_141 = x_235; -x_142 = x_232; +x_140 = x_232; +x_141 = x_234; +x_142 = x_235; x_143 = x_236; x_144 = lean_box(0); goto block_161; @@ -11963,9 +11963,9 @@ lean_inc(x_241); lean_dec(x_236); x_242 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_242, 0, x_241); -x_140 = x_234; -x_141 = x_235; -x_142 = x_232; +x_140 = x_232; +x_141 = x_234; +x_142 = x_235; x_143 = x_242; x_144 = lean_box(0); goto block_161; @@ -11989,9 +11989,9 @@ x_245 = !lean_is_exclusive(x_244); if (x_245 == 0) { lean_ctor_set_tag(x_244, 1); -x_212 = x_234; -x_213 = x_243; -x_214 = x_232; +x_212 = x_232; +x_213 = x_234; +x_214 = x_243; x_215 = x_244; x_216 = lean_box(0); goto block_230; @@ -12004,9 +12004,9 @@ lean_inc(x_246); lean_dec(x_244); x_247 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_247, 0, x_246); -x_212 = x_234; -x_213 = x_243; -x_214 = x_232; +x_212 = x_232; +x_213 = x_234; +x_214 = x_243; x_215 = x_247; x_216 = lean_box(0); goto block_230; @@ -12019,9 +12019,9 @@ x_248 = !lean_is_exclusive(x_244); if (x_248 == 0) { lean_ctor_set_tag(x_244, 0); -x_212 = x_234; -x_213 = x_243; -x_214 = x_232; +x_212 = x_232; +x_213 = x_234; +x_214 = x_243; x_215 = x_244; x_216 = lean_box(0); goto block_230; @@ -12034,9 +12034,9 @@ lean_inc(x_249); lean_dec(x_244); x_250 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_250, 0, x_249); -x_212 = x_234; -x_213 = x_243; -x_214 = x_232; +x_212 = x_232; +x_213 = x_234; +x_214 = x_243; x_215 = x_250; x_216 = lean_box(0); goto block_230; @@ -13568,8 +13568,8 @@ if (x_58 == 0) lean_dec(x_54); lean_dec_ref(x_41); lean_dec(x_4); -x_15 = x_57; -x_16 = x_52; +x_15 = x_52; +x_16 = x_57; x_17 = x_43; x_18 = x_44; x_19 = x_45; @@ -13605,8 +13605,8 @@ x_71 = l_Lean_addTrace___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_In if (lean_obj_tag(x_71) == 0) { lean_dec_ref(x_71); -x_15 = x_57; -x_16 = x_52; +x_15 = x_52; +x_16 = x_57; x_17 = x_43; x_18 = x_44; x_19 = x_45; @@ -13910,7 +13910,7 @@ return x_122; { uint8_t x_23; lean_object* x_24; x_23 = 0; -x_24 = l_Lean_Meta_forallTelescope___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__5___redArg(x_16, x_15, x_23, x_17, x_18, x_19, x_20, x_21); +x_24 = l_Lean_Meta_forallTelescope___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__5___redArg(x_15, x_16, x_23, x_17, x_18, x_19, x_20, x_21); return x_24; } } @@ -16975,7 +16975,7 @@ goto _start; LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__12___redArg___lam__0(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, uint8_t x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* 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; lean_object* x_109; lean_object* x_110; size_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_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_172; lean_object* x_173; uint8_t x_174; +size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_109; lean_object* x_110; lean_object* x_111; size_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_inc(x_1); x_172 = l_Lean_isTracingEnabledFor___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__10___redArg(x_1, x_15); x_173 = lean_ctor_get(x_172, 0); @@ -17053,7 +17053,7 @@ return x_184; { size_t x_26; lean_object* x_27; x_26 = lean_array_size(x_2); -x_27 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__9(x_2, x_26, x_20, x_3, x_21, x_22, x_23, x_24); +x_27 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__9(x_2, x_26, x_18, x_3, x_21, x_22, x_23, x_24); lean_dec_ref(x_2); if (lean_obj_tag(x_27) == 0) { @@ -17065,7 +17065,7 @@ lean_inc(x_24); lean_inc_ref(x_23); lean_inc(x_22); lean_inc_ref(x_21); -x_29 = lean_apply_7(x_4, x_28, x_18, x_21, x_22, x_23, x_24, lean_box(0)); +x_29 = lean_apply_7(x_4, x_28, x_20, x_21, x_22, x_23, x_24, lean_box(0)); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; uint8_t x_31; uint8_t x_32; lean_object* x_33; @@ -17426,8 +17426,8 @@ lean_dec(x_24); lean_dec_ref(x_23); lean_dec(x_22); lean_dec_ref(x_21); +lean_dec_ref(x_20); lean_dec_ref(x_19); -lean_dec_ref(x_18); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_4); @@ -17453,7 +17453,7 @@ return x_107; { lean_object* x_117; uint8_t x_118; lean_inc(x_1); -x_117 = l_Lean_isTracingEnabledFor___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__10___redArg(x_1, x_114); +x_117 = l_Lean_isTracingEnabledFor___at___00Lean_withTraceNode___at___00Lean_Meta_IndPredBelow_mkBelow_spec__8_spec__10___redArg(x_1, x_110); x_118 = !lean_is_exclusive(x_117); if (x_118 == 0) { @@ -17465,13 +17465,13 @@ if (x_120 == 0) { lean_free_object(x_117); lean_dec(x_8); -x_18 = x_116; -x_19 = x_110; -x_20 = x_111; -x_21 = x_109; -x_22 = x_112; -x_23 = x_114; -x_24 = x_113; +x_18 = x_112; +x_19 = x_114; +x_20 = x_116; +x_21 = x_111; +x_22 = x_113; +x_23 = x_110; +x_24 = x_109; x_25 = lean_box(0); goto block_108; } @@ -17490,8 +17490,8 @@ x_125 = l_Array_mapFinIdxM_map___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_sp x_126 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_126, 0, x_124); lean_ctor_set(x_126, 1, x_125); -lean_inc_ref(x_110); -x_127 = lean_array_to_list(x_110); +lean_inc_ref(x_114); +x_127 = lean_array_to_list(x_114); x_128 = lean_box(0); x_129 = l_List_mapTR_loop___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__7(x_127, x_128); x_130 = l_Lean_MessageData_ofList(x_129); @@ -17499,17 +17499,17 @@ x_131 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_131, 0, x_126); lean_ctor_set(x_131, 1, x_130); lean_inc(x_1); -x_132 = l_Lean_addTrace___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__10(x_1, x_131, x_109, x_112, x_114, x_113); +x_132 = l_Lean_addTrace___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__10(x_1, x_131, x_111, x_113, x_110, x_109); if (lean_obj_tag(x_132) == 0) { lean_dec_ref(x_132); -x_18 = x_116; -x_19 = x_110; -x_20 = x_111; -x_21 = x_109; -x_22 = x_112; -x_23 = x_114; -x_24 = x_113; +x_18 = x_112; +x_19 = x_114; +x_20 = x_116; +x_21 = x_111; +x_22 = x_113; +x_23 = x_110; +x_24 = x_109; x_25 = lean_box(0); goto block_108; } @@ -17519,9 +17519,9 @@ uint8_t x_133; lean_dec_ref(x_116); lean_dec_ref(x_114); lean_dec(x_113); -lean_dec(x_112); +lean_dec_ref(x_111); lean_dec_ref(x_110); -lean_dec_ref(x_109); +lean_dec(x_109); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_4); @@ -17557,13 +17557,13 @@ lean_dec(x_136); if (x_137 == 0) { lean_dec(x_8); -x_18 = x_116; -x_19 = x_110; -x_20 = x_111; -x_21 = x_109; -x_22 = x_112; -x_23 = x_114; -x_24 = x_113; +x_18 = x_112; +x_19 = x_114; +x_20 = x_116; +x_21 = x_111; +x_22 = x_113; +x_23 = x_110; +x_24 = x_109; x_25 = lean_box(0); goto block_108; } @@ -17582,8 +17582,8 @@ x_143 = l_Array_mapFinIdxM_map___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_sp x_144 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_144, 0, x_142); lean_ctor_set(x_144, 1, x_143); -lean_inc_ref(x_110); -x_145 = lean_array_to_list(x_110); +lean_inc_ref(x_114); +x_145 = lean_array_to_list(x_114); x_146 = lean_box(0); x_147 = l_List_mapTR_loop___at___00__private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_spec__7(x_145, x_146); x_148 = l_Lean_MessageData_ofList(x_147); @@ -17591,17 +17591,17 @@ x_149 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_149, 0, x_144); lean_ctor_set(x_149, 1, x_148); lean_inc(x_1); -x_150 = l_Lean_addTrace___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__10(x_1, x_149, x_109, x_112, x_114, x_113); +x_150 = l_Lean_addTrace___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__10(x_1, x_149, x_111, x_113, x_110, x_109); if (lean_obj_tag(x_150) == 0) { lean_dec_ref(x_150); -x_18 = x_116; -x_19 = x_110; -x_20 = x_111; -x_21 = x_109; -x_22 = x_112; -x_23 = x_114; -x_24 = x_113; +x_18 = x_112; +x_19 = x_114; +x_20 = x_116; +x_21 = x_111; +x_22 = x_113; +x_23 = x_110; +x_24 = x_109; x_25 = lean_box(0); goto block_108; } @@ -17611,9 +17611,9 @@ lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_dec_ref(x_116); lean_dec_ref(x_114); lean_dec(x_113); -lean_dec(x_112); +lean_dec_ref(x_111); lean_dec_ref(x_110); -lean_dec_ref(x_109); +lean_dec(x_109); lean_dec_ref(x_7); lean_dec(x_6); lean_dec_ref(x_4); @@ -17653,12 +17653,12 @@ lean_inc_ref(x_7); x_165 = l_Lean_Expr_beta(x_7, x_164); if (x_11 == 0) { -x_109 = x_155; -x_110 = x_163; -x_111 = x_162; -x_112 = x_156; -x_113 = x_158; -x_114 = x_157; +x_109 = x_158; +x_110 = x_157; +x_111 = x_155; +x_112 = x_162; +x_113 = x_156; +x_114 = x_163; x_115 = lean_box(0); x_116 = x_165; goto block_154; @@ -17676,24 +17676,24 @@ if (x_168 == 0) lean_object* x_169; lean_object* x_170; x_169 = l_Array_mapFinIdxM_map___at___00Lean_Meta_IndPredBelow_mkBelowMatcher_spec__12___redArg___lam__0___closed__15; x_170 = l_Lean_Expr_betaRev(x_165, x_169, x_5, x_5); -x_109 = x_155; -x_110 = x_163; -x_111 = x_162; -x_112 = x_156; -x_113 = x_158; -x_114 = x_157; +x_109 = x_158; +x_110 = x_157; +x_111 = x_155; +x_112 = x_162; +x_113 = x_156; +x_114 = x_163; x_115 = lean_box(0); x_116 = x_170; goto block_154; } else { -x_109 = x_155; -x_110 = x_163; -x_111 = x_162; -x_112 = x_156; -x_113 = x_158; -x_114 = x_157; +x_109 = x_158; +x_110 = x_157; +x_111 = x_155; +x_112 = x_162; +x_113 = x_156; +x_114 = x_163; x_115 = lean_box(0); x_116 = x_165; goto block_154; @@ -17701,12 +17701,12 @@ goto block_154; } else { -x_109 = x_155; -x_110 = x_163; -x_111 = x_162; -x_112 = x_156; -x_113 = x_158; -x_114 = x_157; +x_109 = x_158; +x_110 = x_157; +x_111 = x_155; +x_112 = x_162; +x_113 = x_156; +x_114 = x_163; x_115 = lean_box(0); x_116 = x_165; goto block_154; diff --git a/stage0/stdlib/Lean/Meta/Injective.c b/stage0/stdlib/Lean/Meta/Injective.c index cab1fc40513c..436d64f503aa 100644 --- a/stage0/stdlib/Lean/Meta/Injective.c +++ b/stage0/stdlib/Lean/Meta/Injective.c @@ -7701,7 +7701,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg(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) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_28; double x_29; lean_object* x_30; lean_object* x_31; double x_32; lean_object* x_33; lean_object* x_34; lean_object* x_39; uint8_t x_40; double x_41; lean_object* x_42; lean_object* x_43; double x_44; 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_64; double x_65; uint8_t x_66; lean_object* x_67; double x_68; lean_object* x_69; lean_object* x_70; lean_object* x_75; double x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; double x_80; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; double x_89; lean_object* x_90; lean_object* x_91; double x_92; uint8_t x_93; lean_object* x_127; uint8_t x_128; double x_129; lean_object* x_130; lean_object* x_131; double x_132; double x_133; lean_object* x_137; uint8_t x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_159; double x_160; lean_object* x_161; uint8_t x_162; lean_object* x_163; double x_164; uint8_t x_165; lean_object* x_199; double x_200; lean_object* x_201; lean_object* x_202; uint8_t x_203; double x_204; double x_205; lean_object* x_209; lean_object* x_210; uint8_t x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; +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; double x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; double x_32; lean_object* x_33; lean_object* x_34; double x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; double x_43; lean_object* x_44; 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_64; double x_65; double x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_75; double x_76; double x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_85; lean_object* x_86; double x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; double x_91; lean_object* x_92; uint8_t x_93; double x_127; lean_object* x_128; uint8_t x_129; lean_object* x_130; double x_131; lean_object* x_132; double x_133; lean_object* x_137; lean_object* x_138; uint8_t x_139; lean_object* x_140; lean_object* x_141; lean_object* x_159; double x_160; double x_161; lean_object* x_162; uint8_t x_163; lean_object* x_164; uint8_t x_165; lean_object* x_199; double x_200; double x_201; lean_object* x_202; lean_object* x_203; uint8_t x_204; double x_205; lean_object* x_209; lean_object* x_210; uint8_t x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; x_11 = lean_ctor_get(x_8, 2); x_12 = lean_ctor_get(x_8, 5); lean_inc(x_1); @@ -7739,7 +7739,7 @@ goto block_248; block_27: { lean_object* x_22; -x_22 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__3(x_13, x_16, x_12, x_15, x_17, x_18, x_19, x_20); +x_22 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__3(x_15, x_16, x_12, x_14, x_17, x_18, x_19, x_20); lean_dec(x_20); lean_dec(x_18); lean_dec_ref(x_17); @@ -7747,13 +7747,13 @@ if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_dec_ref(x_22); -x_23 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_14); +x_23 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_13); return x_23; } else { uint8_t x_24; -lean_dec_ref(x_14); +lean_dec_ref(x_13); x_24 = !lean_is_exclusive(x_22); if (x_24 == 0) { @@ -7773,7 +7773,7 @@ return x_26; } block_38: { -if (x_28 == 0) +if (x_29 == 0) { double x_35; lean_object* x_36; x_35 = l_Lean_addTrace___at___00__private_Lean_Meta_Injective_0__Lean_Meta_solveEqOfCtorEq_spec__2___closed__0; @@ -7784,8 +7784,8 @@ lean_ctor_set_float(x_36, sizeof(void*)*2, x_35); lean_ctor_set_float(x_36, sizeof(void*)*2 + 8, x_35); lean_ctor_set_uint8(x_36, sizeof(void*)*2 + 16, x_4); x_13 = x_30; -x_14 = x_31; -x_15 = x_33; +x_14 = x_33; +x_15 = x_31; x_16 = x_36; x_17 = x_6; x_18 = x_7; @@ -7800,12 +7800,12 @@ lean_object* x_37; x_37 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_37, 0, x_1); lean_ctor_set(x_37, 1, x_5); -lean_ctor_set_float(x_37, sizeof(void*)*2, x_29); -lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_32); +lean_ctor_set_float(x_37, sizeof(void*)*2, x_32); +lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_28); lean_ctor_set_uint8(x_37, sizeof(void*)*2 + 16, x_4); x_13 = x_30; -x_14 = x_31; -x_15 = x_33; +x_14 = x_33; +x_15 = x_31; x_16 = x_37; x_17 = x_6; x_18 = x_7; @@ -7822,19 +7822,19 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_43); -x_45 = lean_apply_6(x_2, x_43, x_6, x_7, x_8, x_9, lean_box(0)); +lean_inc_ref(x_40); +x_45 = lean_apply_6(x_2, x_40, x_6, x_7, x_8, x_9, lean_box(0)); if (lean_obj_tag(x_45) == 0) { lean_object* x_46; x_46 = lean_ctor_get(x_45, 0); lean_inc(x_46); lean_dec_ref(x_45); -x_28 = x_40; +x_28 = x_39; x_29 = x_41; -x_30 = x_42; -x_31 = x_43; -x_32 = x_44; +x_30 = x_40; +x_31 = x_42; +x_32 = x_43; x_33 = x_46; x_34 = lean_box(0); goto block_38; @@ -7844,11 +7844,11 @@ else lean_object* x_47; lean_dec_ref(x_45); x_47 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__1; -x_28 = x_40; +x_28 = x_39; x_29 = x_41; -x_30 = x_42; -x_31 = x_43; -x_32 = x_44; +x_30 = x_40; +x_31 = x_42; +x_32 = x_43; x_33 = x_47; x_34 = lean_box(0); goto block_38; @@ -7857,7 +7857,7 @@ goto block_38; block_63: { lean_object* x_58; -x_58 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__3(x_51, x_52, x_12, x_50, x_53, x_54, x_55, x_56); +x_58 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__3(x_50, x_52, x_12, x_51, x_53, x_54, x_55, x_56); lean_dec(x_56); lean_dec(x_54); lean_dec_ref(x_53); @@ -7891,7 +7891,7 @@ return x_62; } block_74: { -if (x_66 == 0) +if (x_68 == 0) { double x_71; lean_object* x_72; x_71 = l_Lean_addTrace___at___00__private_Lean_Meta_Injective_0__Lean_Meta_solveEqOfCtorEq_spec__2___closed__0; @@ -7902,8 +7902,8 @@ lean_ctor_set_float(x_72, sizeof(void*)*2, x_71); lean_ctor_set_float(x_72, sizeof(void*)*2 + 8, x_71); lean_ctor_set_uint8(x_72, sizeof(void*)*2 + 16, x_4); x_49 = x_64; -x_50 = x_69; -x_51 = x_67; +x_50 = x_67; +x_51 = x_69; x_52 = x_72; x_53 = x_6; x_54 = x_7; @@ -7919,11 +7919,11 @@ x_73 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_73, 0, x_1); lean_ctor_set(x_73, 1, x_5); lean_ctor_set_float(x_73, sizeof(void*)*2, x_65); -lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_68); +lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_66); lean_ctor_set_uint8(x_73, sizeof(void*)*2 + 16, x_4); x_49 = x_64; -x_50 = x_69; -x_51 = x_67; +x_50 = x_67; +x_51 = x_69; x_52 = x_73; x_53 = x_6; x_54 = x_7; @@ -7950,7 +7950,7 @@ lean_inc(x_82); lean_dec_ref(x_81); x_64 = x_75; x_65 = x_76; -x_66 = x_79; +x_66 = x_77; x_67 = x_78; x_68 = x_80; x_69 = x_82; @@ -7964,7 +7964,7 @@ lean_dec_ref(x_81); x_83 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__1; x_64 = x_75; x_65 = x_76; -x_66 = x_79; +x_66 = x_77; x_67 = x_78; x_68 = x_80; x_69 = x_83; @@ -8005,7 +8005,7 @@ lean_dec_ref(x_99); lean_ctor_set(x_97, 0, x_100); x_101 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_91); +x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_89); return x_102; } else @@ -8023,7 +8023,7 @@ lean_ctor_set_uint64(x_106, sizeof(void*)*1, x_103); lean_ctor_set(x_95, 4, x_106); x_107 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_91); +x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_89); return x_108; } } @@ -8080,43 +8080,43 @@ lean_ctor_set(x_123, 7, x_116); lean_ctor_set(x_123, 8, x_117); x_124 = lean_st_ref_set(x_9, x_123); lean_dec(x_9); -x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_91); +x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__4___redArg(x_89); return x_125; } } else { -x_39 = lean_box(0); -x_40 = x_88; -x_41 = x_89; +x_39 = x_87; +x_40 = x_89; +x_41 = x_88; x_42 = x_90; x_43 = x_91; -x_44 = x_92; +x_44 = lean_box(0); goto block_48; } } else { -x_39 = lean_box(0); -x_40 = x_88; -x_41 = x_89; +x_39 = x_87; +x_40 = x_89; +x_41 = x_88; x_42 = x_90; x_43 = x_91; -x_44 = x_92; +x_44 = lean_box(0); goto block_48; } } block_136: { double x_134; uint8_t x_135; -x_134 = lean_float_sub(x_132, x_129); +x_134 = lean_float_sub(x_127, x_131); x_135 = lean_float_decLt(x_133, x_134); -x_87 = lean_box(0); -x_88 = x_128; -x_89 = x_129; +x_87 = x_127; +x_88 = x_129; +x_89 = x_128; x_90 = x_130; x_91 = x_131; -x_92 = x_132; +x_92 = lean_box(0); x_93 = x_135; goto block_126; } @@ -8124,7 +8124,7 @@ goto block_126; { lean_object* x_142; double x_143; double x_144; double x_145; double x_146; double x_147; lean_object* x_148; uint8_t x_149; x_142 = lean_io_mono_nanos_now(); -x_143 = lean_float_of_nat(x_139); +x_143 = lean_float_of_nat(x_138); x_144 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__2; x_145 = lean_float_div(x_143, x_144); x_146 = lean_float_of_nat(x_142); @@ -8133,18 +8133,18 @@ x_148 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta x_149 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__2(x_11, x_148); if (x_149 == 0) { -x_87 = lean_box(0); +x_87 = x_147; x_88 = x_149; -x_89 = x_145; +x_89 = x_140; x_90 = x_137; -x_91 = x_140; -x_92 = x_147; +x_91 = x_145; +x_92 = lean_box(0); x_93 = x_149; goto block_126; } else { -if (x_138 == 0) +if (x_139 == 0) { lean_object* x_150; lean_object* x_151; double x_152; double x_153; double x_154; x_150 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__4; @@ -8152,12 +8152,12 @@ x_151 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Me x_152 = lean_float_of_nat(x_151); x_153 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__5; x_154 = lean_float_div(x_152, x_153); -x_127 = lean_box(0); -x_128 = x_149; -x_129 = x_145; +x_127 = x_147; +x_128 = x_140; +x_129 = x_149; x_130 = x_137; -x_131 = x_140; -x_132 = x_147; +x_131 = x_145; +x_132 = lean_box(0); x_133 = x_154; goto block_136; } @@ -8167,12 +8167,12 @@ lean_object* x_155; lean_object* x_156; double x_157; x_155 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1___redArg___closed__4; x_156 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheorem_spec__1_spec__5(x_11, x_155); x_157 = lean_float_of_nat(x_156); -x_127 = lean_box(0); -x_128 = x_149; -x_129 = x_145; +x_127 = x_147; +x_128 = x_140; +x_129 = x_149; x_130 = x_137; -x_131 = x_140; -x_132 = x_147; +x_131 = x_145; +x_132 = lean_box(0); x_133 = x_157; goto block_136; } @@ -8206,7 +8206,7 @@ if (x_170 == 0) { lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; x_171 = lean_ctor_get(x_169, 0); -x_172 = l_Lean_PersistentArray_append___redArg(x_163, x_171); +x_172 = l_Lean_PersistentArray_append___redArg(x_162, x_171); lean_dec_ref(x_171); lean_ctor_set(x_169, 0, x_172); x_173 = lean_st_ref_set(x_9, x_167); @@ -8221,7 +8221,7 @@ x_175 = lean_ctor_get_uint64(x_169, sizeof(void*)*1); x_176 = lean_ctor_get(x_169, 0); lean_inc(x_176); lean_dec(x_169); -x_177 = l_Lean_PersistentArray_append___redArg(x_163, x_176); +x_177 = l_Lean_PersistentArray_append___redArg(x_162, x_176); lean_dec_ref(x_176); x_178 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_178, 0, x_177); @@ -8265,7 +8265,7 @@ if (lean_is_exclusive(x_181)) { lean_dec_ref(x_181); x_192 = lean_box(0); } -x_193 = l_Lean_PersistentArray_append___redArg(x_163, x_191); +x_193 = l_Lean_PersistentArray_append___redArg(x_162, x_191); lean_dec_ref(x_191); if (lean_is_scalar(x_192)) { x_194 = lean_alloc_ctor(0, 1, 8); @@ -8294,10 +8294,10 @@ else { x_75 = x_159; x_76 = x_160; -x_77 = lean_box(0); -x_78 = x_163; -x_79 = x_162; -x_80 = x_164; +x_77 = x_161; +x_78 = x_162; +x_79 = lean_box(0); +x_80 = x_163; goto block_84; } } @@ -8305,24 +8305,24 @@ else { x_75 = x_159; x_76 = x_160; -x_77 = lean_box(0); -x_78 = x_163; -x_79 = x_162; -x_80 = x_164; +x_77 = x_161; +x_78 = x_162; +x_79 = lean_box(0); +x_80 = x_163; goto block_84; } } block_208: { double x_206; uint8_t x_207; -x_206 = lean_float_sub(x_204, x_200); +x_206 = lean_float_sub(x_201, x_200); x_207 = lean_float_decLt(x_205, x_206); x_159 = x_199; x_160 = x_200; -x_161 = lean_box(0); -x_162 = x_203; -x_163 = x_202; -x_164 = x_204; +x_161 = x_201; +x_162 = x_202; +x_163 = x_204; +x_164 = lean_box(0); x_165 = x_207; goto block_198; } @@ -8338,10 +8338,10 @@ if (x_218 == 0) { x_159 = x_212; x_160 = x_215; -x_161 = lean_box(0); -x_162 = x_218; -x_163 = x_210; -x_164 = x_216; +x_161 = x_216; +x_162 = x_210; +x_163 = x_218; +x_164 = lean_box(0); x_165 = x_218; goto block_198; } @@ -8357,10 +8357,10 @@ x_222 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Injective_0__Lean_Meta x_223 = lean_float_div(x_221, x_222); x_199 = x_212; x_200 = x_215; -x_201 = lean_box(0); +x_201 = x_216; x_202 = x_210; -x_203 = x_218; -x_204 = x_216; +x_203 = lean_box(0); +x_204 = x_218; x_205 = x_223; goto block_208; } @@ -8372,10 +8372,10 @@ x_225 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Me x_226 = lean_float_of_nat(x_225); x_199 = x_212; x_200 = x_215; -x_201 = lean_box(0); +x_201 = x_216; x_202 = x_210; -x_203 = x_218; -x_204 = x_216; +x_203 = lean_box(0); +x_204 = x_218; x_205 = x_226; goto block_208; } @@ -8407,8 +8407,8 @@ if (x_234 == 0) { lean_ctor_set_tag(x_233, 1); x_137 = x_229; -x_138 = x_231; -x_139 = x_232; +x_138 = x_232; +x_139 = x_231; x_140 = x_233; x_141 = lean_box(0); goto block_158; @@ -8422,8 +8422,8 @@ lean_dec(x_233); x_236 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_236, 0, x_235); x_137 = x_229; -x_138 = x_231; -x_139 = x_232; +x_138 = x_232; +x_139 = x_231; x_140 = x_236; x_141 = lean_box(0); goto block_158; @@ -8437,8 +8437,8 @@ if (x_237 == 0) { lean_ctor_set_tag(x_233, 0); x_137 = x_229; -x_138 = x_231; -x_139 = x_232; +x_138 = x_232; +x_139 = x_231; x_140 = x_233; x_141 = lean_box(0); goto block_158; @@ -8452,8 +8452,8 @@ lean_dec(x_233); x_239 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_239, 0, x_238); x_137 = x_229; -x_138 = x_231; -x_139 = x_232; +x_138 = x_232; +x_139 = x_231; x_140 = x_239; x_141 = lean_box(0); goto block_158; diff --git a/stage0/stdlib/Lean/Meta/LazyDiscrTree.c b/stage0/stdlib/Lean/Meta/LazyDiscrTree.c index cb90e3dff126..6117f78951f6 100644 --- a/stage0/stdlib/Lean/Meta/LazyDiscrTree.c +++ b/stage0/stdlib/Lean/Meta/LazyDiscrTree.c @@ -18462,7 +18462,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createImportedDiscrTree___at___00Lean_Meta_LazyDiscrTree_findImportMatches_spec__0_spec__0_spec__2_spec__3_spec__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) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t 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_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; uint8_t x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t 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_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; uint8_t x_94; uint8_t x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; uint8_t x_109; uint8_t x_125; x_100 = 2; x_125 = l_Lean_instBEqMessageSeverity_beq(x_3, x_100); if (x_125 == 0) @@ -18497,15 +18497,15 @@ lean_ctor_set(x_25, 0, x_21); lean_ctor_set(x_25, 1, x_22); x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_10); +lean_ctor_set(x_26, 1, x_14); x_27 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_27, 0, x_13); -lean_ctor_set(x_27, 1, x_16); +lean_ctor_set(x_27, 0, x_10); +lean_ctor_set(x_27, 1, x_12); lean_ctor_set(x_27, 2, x_11); -lean_ctor_set(x_27, 3, x_14); +lean_ctor_set(x_27, 3, x_16); lean_ctor_set(x_27, 4, x_26); lean_ctor_set_uint8(x_27, sizeof(void*)*5, x_15); -lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_12); +lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 1, x_13); lean_ctor_set_uint8(x_27, sizeof(void*)*5 + 2, x_4); x_28 = l_Lean_MessageLog_add(x_27, x_24); lean_ctor_set(x_20, 6, x_28); @@ -18542,15 +18542,15 @@ lean_ctor_set(x_41, 0, x_21); lean_ctor_set(x_41, 1, x_22); x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_10); +lean_ctor_set(x_42, 1, x_14); x_43 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_43, 0, x_13); -lean_ctor_set(x_43, 1, x_16); +lean_ctor_set(x_43, 0, x_10); +lean_ctor_set(x_43, 1, x_12); lean_ctor_set(x_43, 2, x_11); -lean_ctor_set(x_43, 3, x_14); +lean_ctor_set(x_43, 3, x_16); lean_ctor_set(x_43, 4, x_42); lean_ctor_set_uint8(x_43, sizeof(void*)*5, x_15); -lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_12); +lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 1, x_13); lean_ctor_set_uint8(x_43, sizeof(void*)*5 + 2, x_4); x_44 = l_Lean_MessageLog_add(x_43, x_38); x_45 = lean_alloc_ctor(0, 9, 0); @@ -18581,24 +18581,24 @@ if (x_60 == 0) lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_61 = lean_ctor_get(x_59, 0); lean_inc_ref(x_55); -x_62 = l_Lean_FileMap_toPosition(x_55, x_52); -lean_dec(x_52); +x_62 = l_Lean_FileMap_toPosition(x_55, x_53); +lean_dec(x_53); x_63 = l_Lean_FileMap_toPosition(x_55, x_57); lean_dec(x_57); x_64 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_64, 0, x_63); x_65 = l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createImportedDiscrTree___at___00Lean_Meta_LazyDiscrTree_findImportMatches_spec__0_spec__0_spec__2_spec__3_spec__7___closed__0; -if (x_56 == 0) +if (x_51 == 0) { lean_free_object(x_59); lean_dec_ref(x_50); -x_10 = x_61; +x_10 = x_52; x_11 = x_64; -x_12 = x_51; -x_13 = x_53; -x_14 = x_65; -x_15 = x_54; -x_16 = x_62; +x_12 = x_62; +x_13 = x_54; +x_14 = x_61; +x_15 = x_56; +x_16 = x_65; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -18615,7 +18615,7 @@ lean_object* x_67; lean_dec_ref(x_64); lean_dec_ref(x_62); lean_dec(x_61); -lean_dec_ref(x_53); +lean_dec_ref(x_52); lean_dec_ref(x_7); x_67 = lean_box(0); lean_ctor_set(x_59, 0, x_67); @@ -18624,13 +18624,13 @@ return x_59; else { lean_free_object(x_59); -x_10 = x_61; +x_10 = x_52; x_11 = x_64; -x_12 = x_51; -x_13 = x_53; -x_14 = x_65; -x_15 = x_54; -x_16 = x_62; +x_12 = x_62; +x_13 = x_54; +x_14 = x_61; +x_15 = x_56; +x_16 = x_65; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -18645,23 +18645,23 @@ x_68 = lean_ctor_get(x_59, 0); lean_inc(x_68); lean_dec(x_59); lean_inc_ref(x_55); -x_69 = l_Lean_FileMap_toPosition(x_55, x_52); -lean_dec(x_52); +x_69 = l_Lean_FileMap_toPosition(x_55, x_53); +lean_dec(x_53); x_70 = l_Lean_FileMap_toPosition(x_55, x_57); lean_dec(x_57); x_71 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_71, 0, x_70); x_72 = l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createImportedDiscrTree___at___00Lean_Meta_LazyDiscrTree_findImportMatches_spec__0_spec__0_spec__2_spec__3_spec__7___closed__0; -if (x_56 == 0) +if (x_51 == 0) { lean_dec_ref(x_50); -x_10 = x_68; +x_10 = x_52; x_11 = x_71; -x_12 = x_51; -x_13 = x_53; -x_14 = x_72; -x_15 = x_54; -x_16 = x_69; +x_12 = x_69; +x_13 = x_54; +x_14 = x_68; +x_15 = x_56; +x_16 = x_72; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -18678,7 +18678,7 @@ lean_object* x_74; lean_object* x_75; lean_dec_ref(x_71); lean_dec_ref(x_69); lean_dec(x_68); -lean_dec_ref(x_53); +lean_dec_ref(x_52); lean_dec_ref(x_7); x_74 = lean_box(0); x_75 = lean_alloc_ctor(0, 1, 0); @@ -18687,13 +18687,13 @@ return x_75; } else { -x_10 = x_68; +x_10 = x_52; x_11 = x_71; -x_12 = x_51; -x_13 = x_53; -x_14 = x_72; -x_15 = x_54; -x_16 = x_69; +x_12 = x_69; +x_13 = x_54; +x_14 = x_68; +x_15 = x_56; +x_16 = x_72; x_17 = x_7; x_18 = x_8; x_19 = lean_box(0); @@ -18705,18 +18705,18 @@ goto block_49; block_87: { lean_object* x_85; -x_85 = l_Lean_Syntax_getTailPos_x3f(x_82, x_81); -lean_dec(x_82); +x_85 = l_Lean_Syntax_getTailPos_x3f(x_83, x_82); +lean_dec(x_83); if (lean_obj_tag(x_85) == 0) { lean_inc(x_84); x_50 = x_77; -x_51 = x_78; -x_52 = x_84; -x_53 = x_79; -x_54 = x_81; -x_55 = x_80; -x_56 = x_83; +x_51 = x_79; +x_52 = x_78; +x_53 = x_84; +x_54 = x_80; +x_55 = x_81; +x_56 = x_82; x_57 = x_84; goto block_76; } @@ -18727,12 +18727,12 @@ x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); lean_dec_ref(x_85); x_50 = x_77; -x_51 = x_78; -x_52 = x_84; -x_53 = x_79; -x_54 = x_81; -x_55 = x_80; -x_56 = x_83; +x_51 = x_79; +x_52 = x_78; +x_53 = x_84; +x_54 = x_80; +x_55 = x_81; +x_56 = x_82; x_57 = x_86; goto block_76; } @@ -18740,20 +18740,20 @@ goto block_76; block_99: { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_replaceRef(x_1, x_90); -lean_dec(x_90); -x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_91); +x_95 = l_Lean_replaceRef(x_1, x_91); +lean_dec(x_91); +x_96 = l_Lean_Syntax_getPos_x3f(x_95, x_93); if (lean_obj_tag(x_96) == 0) { lean_object* x_97; x_97 = lean_unsigned_to_nat(0u); x_77 = x_88; -x_78 = x_94; +x_78 = x_90; x_79 = x_89; -x_80 = x_92; -x_81 = x_91; -x_82 = x_95; -x_83 = x_93; +x_80 = x_94; +x_81 = x_92; +x_82 = x_93; +x_83 = x_95; x_84 = x_97; goto block_87; } @@ -18764,12 +18764,12 @@ x_98 = lean_ctor_get(x_96, 0); lean_inc(x_98); lean_dec_ref(x_96); x_77 = x_88; -x_78 = x_94; +x_78 = x_90; x_79 = x_89; -x_80 = x_92; -x_81 = x_91; -x_82 = x_95; -x_83 = x_93; +x_80 = x_94; +x_81 = x_92; +x_82 = x_93; +x_83 = x_95; x_84 = x_98; goto block_87; } @@ -18778,23 +18778,23 @@ goto block_87; { if (x_107 == 0) { -x_88 = x_101; +x_88 = x_105; x_89 = x_102; -x_90 = x_103; -x_91 = x_106; +x_90 = x_101; +x_91 = x_103; x_92 = x_104; -x_93 = x_105; +x_93 = x_106; x_94 = x_3; goto block_99; } else { -x_88 = x_101; +x_88 = x_105; x_89 = x_102; -x_90 = x_103; -x_91 = x_106; +x_90 = x_101; +x_91 = x_103; x_92 = x_104; -x_93 = x_105; +x_93 = x_106; x_94 = x_100; goto block_99; } @@ -18821,11 +18821,11 @@ if (x_119 == 0) lean_inc_ref(x_111); lean_inc(x_113); lean_inc_ref(x_110); -x_101 = x_117; -x_102 = x_110; +x_101 = x_110; +x_102 = x_114; x_103 = x_113; x_104 = x_111; -x_105 = x_114; +x_105 = x_117; x_106 = x_109; x_107 = x_119; goto block_108; @@ -18838,11 +18838,11 @@ x_121 = l_Lean_Option_get___at___00Lean_Meta_LazyDiscrTree_addConstImportData_sp lean_inc_ref(x_111); lean_inc(x_113); lean_inc_ref(x_110); -x_101 = x_117; -x_102 = x_110; +x_101 = x_110; +x_102 = x_114; x_103 = x_113; x_104 = x_111; -x_105 = x_114; +x_105 = x_117; x_106 = x_109; x_107 = x_121; goto block_108; @@ -20279,7 +20279,7 @@ return x_12; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createModuleDiscrTree_spec__0_spec__0_spec__2_spec__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -uint8_t 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_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; uint8_t x_91; uint8_t x_92; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; uint8_t x_104; uint8_t x_105; uint8_t x_107; uint8_t x_123; +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; uint8_t x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_75; lean_object* x_76; uint8_t x_77; uint8_t x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; uint8_t x_92; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; uint8_t x_104; uint8_t x_105; uint8_t x_107; uint8_t x_123; x_98 = 2; x_123 = l_Lean_instBEqMessageSeverity_beq(x_3, x_98); if (x_123 == 0) @@ -20314,15 +20314,15 @@ lean_ctor_set(x_23, 0, x_19); lean_ctor_set(x_23, 1, x_20); x_24 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_10); +lean_ctor_set(x_24, 1, x_9); x_25 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_25, 0, x_9); -lean_ctor_set(x_25, 1, x_12); -lean_ctor_set(x_25, 2, x_13); -lean_ctor_set(x_25, 3, x_14); +lean_ctor_set(x_25, 0, x_13); +lean_ctor_set(x_25, 1, x_14); +lean_ctor_set(x_25, 2, x_10); +lean_ctor_set(x_25, 3, x_8); lean_ctor_set(x_25, 4, x_24); -lean_ctor_set_uint8(x_25, sizeof(void*)*5, x_11); -lean_ctor_set_uint8(x_25, sizeof(void*)*5 + 1, x_8); +lean_ctor_set_uint8(x_25, sizeof(void*)*5, x_12); +lean_ctor_set_uint8(x_25, sizeof(void*)*5 + 1, x_11); lean_ctor_set_uint8(x_25, sizeof(void*)*5 + 2, x_4); x_26 = l_Lean_MessageLog_add(x_25, x_22); lean_ctor_set(x_18, 6, x_26); @@ -20359,15 +20359,15 @@ lean_ctor_set(x_39, 0, x_19); lean_ctor_set(x_39, 1, x_20); x_40 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_10); +lean_ctor_set(x_40, 1, x_9); x_41 = lean_alloc_ctor(0, 5, 3); -lean_ctor_set(x_41, 0, x_9); -lean_ctor_set(x_41, 1, x_12); -lean_ctor_set(x_41, 2, x_13); -lean_ctor_set(x_41, 3, x_14); +lean_ctor_set(x_41, 0, x_13); +lean_ctor_set(x_41, 1, x_14); +lean_ctor_set(x_41, 2, x_10); +lean_ctor_set(x_41, 3, x_8); lean_ctor_set(x_41, 4, x_40); -lean_ctor_set_uint8(x_41, sizeof(void*)*5, x_11); -lean_ctor_set_uint8(x_41, sizeof(void*)*5 + 1, x_8); +lean_ctor_set_uint8(x_41, sizeof(void*)*5, x_12); +lean_ctor_set_uint8(x_41, sizeof(void*)*5 + 1, x_11); lean_ctor_set_uint8(x_41, sizeof(void*)*5 + 2, x_4); x_42 = l_Lean_MessageLog_add(x_41, x_36); x_43 = lean_alloc_ctor(0, 9, 0); @@ -20397,25 +20397,25 @@ if (x_58 == 0) { lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; x_59 = lean_ctor_get(x_57, 0); -lean_inc_ref(x_51); -x_60 = l_Lean_FileMap_toPosition(x_51, x_53); -lean_dec(x_53); -x_61 = l_Lean_FileMap_toPosition(x_51, x_55); +lean_inc_ref(x_50); +x_60 = l_Lean_FileMap_toPosition(x_50, x_49); +lean_dec(x_49); +x_61 = l_Lean_FileMap_toPosition(x_50, x_55); lean_dec(x_55); x_62 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_62, 0, x_61); x_63 = l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createImportedDiscrTree___at___00Lean_Meta_LazyDiscrTree_findImportMatches_spec__0_spec__0_spec__2_spec__3_spec__7___closed__0; -if (x_52 == 0) +if (x_54 == 0) { lean_free_object(x_57); lean_dec_ref(x_48); -x_8 = x_50; -x_9 = x_49; -x_10 = x_59; -x_11 = x_54; -x_12 = x_60; -x_13 = x_62; -x_14 = x_63; +x_8 = x_63; +x_9 = x_59; +x_10 = x_62; +x_11 = x_51; +x_12 = x_52; +x_13 = x_53; +x_14 = x_60; x_15 = x_5; x_16 = x_6; x_17 = lean_box(0); @@ -20432,7 +20432,7 @@ lean_object* x_65; lean_dec_ref(x_62); lean_dec_ref(x_60); lean_dec(x_59); -lean_dec_ref(x_49); +lean_dec_ref(x_53); lean_dec_ref(x_5); x_65 = lean_box(0); lean_ctor_set(x_57, 0, x_65); @@ -20441,13 +20441,13 @@ return x_57; else { lean_free_object(x_57); -x_8 = x_50; -x_9 = x_49; -x_10 = x_59; -x_11 = x_54; -x_12 = x_60; -x_13 = x_62; -x_14 = x_63; +x_8 = x_63; +x_9 = x_59; +x_10 = x_62; +x_11 = x_51; +x_12 = x_52; +x_13 = x_53; +x_14 = x_60; x_15 = x_5; x_16 = x_6; x_17 = lean_box(0); @@ -20461,24 +20461,24 @@ lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean x_66 = lean_ctor_get(x_57, 0); lean_inc(x_66); lean_dec(x_57); -lean_inc_ref(x_51); -x_67 = l_Lean_FileMap_toPosition(x_51, x_53); -lean_dec(x_53); -x_68 = l_Lean_FileMap_toPosition(x_51, x_55); +lean_inc_ref(x_50); +x_67 = l_Lean_FileMap_toPosition(x_50, x_49); +lean_dec(x_49); +x_68 = l_Lean_FileMap_toPosition(x_50, x_55); lean_dec(x_55); x_69 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_69, 0, x_68); x_70 = l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_LazyDiscrTree_logImportFailure___at___00Lean_Meta_LazyDiscrTree_createImportedDiscrTree___at___00Lean_Meta_LazyDiscrTree_findImportMatches_spec__0_spec__0_spec__2_spec__3_spec__7___closed__0; -if (x_52 == 0) +if (x_54 == 0) { lean_dec_ref(x_48); -x_8 = x_50; -x_9 = x_49; -x_10 = x_66; -x_11 = x_54; -x_12 = x_67; -x_13 = x_69; -x_14 = x_70; +x_8 = x_70; +x_9 = x_66; +x_10 = x_69; +x_11 = x_51; +x_12 = x_52; +x_13 = x_53; +x_14 = x_67; x_15 = x_5; x_16 = x_6; x_17 = lean_box(0); @@ -20495,7 +20495,7 @@ lean_object* x_72; lean_object* x_73; lean_dec_ref(x_69); lean_dec_ref(x_67); lean_dec(x_66); -lean_dec_ref(x_49); +lean_dec_ref(x_53); lean_dec_ref(x_5); x_72 = lean_box(0); x_73 = lean_alloc_ctor(0, 1, 0); @@ -20504,13 +20504,13 @@ return x_73; } else { -x_8 = x_50; -x_9 = x_49; -x_10 = x_66; -x_11 = x_54; -x_12 = x_67; -x_13 = x_69; -x_14 = x_70; +x_8 = x_70; +x_9 = x_66; +x_10 = x_69; +x_11 = x_51; +x_12 = x_52; +x_13 = x_53; +x_14 = x_67; x_15 = x_5; x_16 = x_6; x_17 = lean_box(0); @@ -20522,17 +20522,17 @@ goto block_47; block_85: { lean_object* x_83; -x_83 = l_Lean_Syntax_getTailPos_x3f(x_81, x_80); +x_83 = l_Lean_Syntax_getTailPos_x3f(x_81, x_78); lean_dec(x_81); if (lean_obj_tag(x_83) == 0) { lean_inc(x_82); x_48 = x_75; -x_49 = x_78; -x_50 = x_77; -x_51 = x_76; -x_52 = x_79; -x_53 = x_82; +x_49 = x_82; +x_50 = x_76; +x_51 = x_77; +x_52 = x_78; +x_53 = x_79; x_54 = x_80; x_55 = x_82; goto block_74; @@ -20544,11 +20544,11 @@ x_84 = lean_ctor_get(x_83, 0); lean_inc(x_84); lean_dec_ref(x_83); x_48 = x_75; -x_49 = x_78; -x_50 = x_77; -x_51 = x_76; -x_52 = x_79; -x_53 = x_82; +x_49 = x_82; +x_50 = x_76; +x_51 = x_77; +x_52 = x_78; +x_53 = x_79; x_54 = x_80; x_55 = x_84; goto block_74; @@ -20557,18 +20557,18 @@ goto block_74; block_97: { lean_object* x_93; lean_object* x_94; -x_93 = l_Lean_replaceRef(x_1, x_89); -lean_dec(x_89); -x_94 = l_Lean_Syntax_getPos_x3f(x_93, x_91); +x_93 = l_Lean_replaceRef(x_1, x_90); +lean_dec(x_90); +x_94 = l_Lean_Syntax_getPos_x3f(x_93, x_88); if (lean_obj_tag(x_94) == 0) { lean_object* x_95; x_95 = lean_unsigned_to_nat(0u); x_75 = x_86; -x_76 = x_88; +x_76 = x_87; x_77 = x_92; -x_78 = x_87; -x_79 = x_90; +x_78 = x_88; +x_79 = x_89; x_80 = x_91; x_81 = x_93; x_82 = x_95; @@ -20581,10 +20581,10 @@ x_96 = lean_ctor_get(x_94, 0); lean_inc(x_96); lean_dec_ref(x_94); x_75 = x_86; -x_76 = x_88; +x_76 = x_87; x_77 = x_92; -x_78 = x_87; -x_79 = x_90; +x_78 = x_88; +x_79 = x_89; x_80 = x_91; x_81 = x_93; x_82 = x_96; @@ -20595,23 +20595,23 @@ goto block_85; { if (x_105 == 0) { -x_86 = x_99; -x_87 = x_101; -x_88 = x_100; -x_89 = x_102; -x_90 = x_103; -x_91 = x_104; +x_86 = x_101; +x_87 = x_99; +x_88 = x_104; +x_89 = x_100; +x_90 = x_102; +x_91 = x_103; x_92 = x_3; goto block_97; } else { -x_86 = x_99; -x_87 = x_101; -x_88 = x_100; -x_89 = x_102; -x_90 = x_103; -x_91 = x_104; +x_86 = x_101; +x_87 = x_99; +x_88 = x_104; +x_89 = x_100; +x_90 = x_102; +x_91 = x_103; x_92 = x_98; goto block_97; } @@ -20638,9 +20638,9 @@ if (x_117 == 0) lean_inc(x_111); lean_inc_ref(x_108); lean_inc_ref(x_109); -x_99 = x_115; -x_100 = x_109; -x_101 = x_108; +x_99 = x_109; +x_100 = x_108; +x_101 = x_115; x_102 = x_111; x_103 = x_112; x_104 = x_107; @@ -20655,9 +20655,9 @@ x_119 = l_Lean_Option_get___at___00Lean_Meta_LazyDiscrTree_addConstImportData_sp lean_inc(x_111); lean_inc_ref(x_108); lean_inc_ref(x_109); -x_99 = x_115; -x_100 = x_109; -x_101 = x_108; +x_99 = x_109; +x_100 = x_108; +x_101 = x_115; x_102 = x_111; x_103 = x_112; x_104 = x_107; diff --git a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c index 0bb65a90ad7f..cdcef417b1b1 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c @@ -9709,15 +9709,15 @@ x_33 = l_Lean_Syntax_getArg(x_29, x_14); lean_dec(x_29); x_34 = l_Lean_Elab_Tactic_expandLocation(x_33); lean_dec(x_33); -x_15 = x_7; -x_16 = x_4; -x_17 = x_2; -x_18 = x_5; -x_19 = x_8; -x_20 = x_3; -x_21 = lean_box(0); -x_22 = x_9; -x_23 = x_6; +x_15 = x_9; +x_16 = x_8; +x_17 = x_5; +x_18 = x_3; +x_19 = lean_box(0); +x_20 = x_7; +x_21 = x_6; +x_22 = x_4; +x_23 = x_2; x_24 = x_34; goto block_27; } @@ -9730,15 +9730,15 @@ x_35 = l_Lean_Meta_AC_evalNf0___closed__2; x_36 = lean_alloc_ctor(1, 1, 1); lean_ctor_set(x_36, 0, x_35); lean_ctor_set_uint8(x_36, sizeof(void*)*1, x_12); -x_15 = x_7; -x_16 = x_4; -x_17 = x_2; -x_18 = x_5; -x_19 = x_8; -x_20 = x_3; -x_21 = lean_box(0); -x_22 = x_9; -x_23 = x_6; +x_15 = x_9; +x_16 = x_8; +x_17 = x_5; +x_18 = x_3; +x_19 = lean_box(0); +x_20 = x_7; +x_21 = x_6; +x_22 = x_4; +x_23 = x_2; x_24 = x_36; goto block_27; } @@ -9748,7 +9748,7 @@ lean_object* x_25; lean_object* x_26; x_25 = lean_alloc_closure((void*)(l_Lean_Meta_AC_evalNf0___lam__0___boxed), 11, 2); lean_closure_set(x_25, 0, x_24); lean_closure_set(x_25, 1, x_14); -x_26 = l_Lean_Elab_Tactic_withMainContext___redArg(x_25, x_17, x_20, x_16, x_18, x_23, x_15, x_19, x_22); +x_26 = l_Lean_Elab_Tactic_withMainContext___redArg(x_25, x_23, x_18, x_22, x_17, x_21, x_20, x_16, x_15); return x_26; } } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Apply.c b/stage0/stdlib/Lean/Meta/Tactic/Apply.c index fe06a27b0f7b..037bfdf227cf 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Apply.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Apply.c @@ -5358,7 +5358,7 @@ goto _start; LEAN_EXPORT lean_object* l_Lean_MVarId_apply___lam__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, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_52; +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_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_52; lean_inc(x_2); lean_inc(x_1); x_52 = l_Lean_MVarId_checkNotAssigned(x_1, x_2, x_6, x_7, x_8, x_9); @@ -5664,13 +5664,13 @@ x_79 = lean_nat_dec_lt(x_76, x_77); if (x_79 == 0) { lean_dec(x_66); -x_28 = x_76; -x_29 = x_60; -x_30 = x_62; -x_31 = x_73; -x_32 = x_61; -x_33 = x_68; -x_34 = x_59; +x_28 = x_68; +x_29 = x_76; +x_30 = x_61; +x_31 = x_62; +x_32 = x_60; +x_33 = x_59; +x_34 = x_73; x_35 = x_78; x_36 = lean_box(0); goto block_51; @@ -5682,13 +5682,13 @@ x_80 = lean_nat_dec_le(x_77, x_77); if (x_80 == 0) { lean_dec(x_66); -x_28 = x_76; -x_29 = x_60; -x_30 = x_62; -x_31 = x_73; -x_32 = x_61; -x_33 = x_68; -x_34 = x_59; +x_28 = x_68; +x_29 = x_76; +x_30 = x_61; +x_31 = x_62; +x_32 = x_60; +x_33 = x_59; +x_34 = x_73; x_35 = x_78; x_36 = lean_box(0); goto block_51; @@ -5706,13 +5706,13 @@ lean_object* x_84; x_84 = lean_ctor_get(x_83, 0); lean_inc(x_84); lean_dec_ref(x_83); -x_28 = x_76; -x_29 = x_60; -x_30 = x_62; -x_31 = x_73; -x_32 = x_61; -x_33 = x_68; -x_34 = x_59; +x_28 = x_68; +x_29 = x_76; +x_30 = x_61; +x_31 = x_62; +x_32 = x_60; +x_33 = x_59; +x_34 = x_73; x_35 = x_84; x_36 = lean_box(0); goto block_51; @@ -5889,11 +5889,11 @@ lean_object* x_18; lean_object* x_19; lean_object* x_20; x_18 = lean_array_to_list(x_17); x_19 = l_List_appendTR___redArg(x_15, x_18); lean_inc(x_19); -x_20 = l_List_forM___at___00Lean_MVarId_apply_spec__3(x_19, x_16, x_11, x_14, x_12); +x_20 = l_List_forM___at___00Lean_MVarId_apply_spec__3(x_19, x_14, x_13, x_11, x_12); lean_dec(x_12); +lean_dec_ref(x_11); +lean_dec(x_13); lean_dec_ref(x_14); -lean_dec(x_11); -lean_dec_ref(x_16); if (lean_obj_tag(x_20) == 0) { uint8_t x_21; @@ -5939,18 +5939,18 @@ return x_26; block_51: { lean_object* x_37; -x_37 = l_Lean_Meta_getMVarsNoDelayed(x_31, x_34, x_29, x_32, x_30); +x_37 = l_Lean_Meta_getMVarsNoDelayed(x_34, x_33, x_32, x_30, x_31); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; lean_object* x_39; x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); lean_dec_ref(x_37); -lean_inc(x_30); -lean_inc_ref(x_32); -lean_inc(x_29); -lean_inc_ref(x_34); -x_39 = l___private_Lean_Meta_Tactic_Apply_0__Lean_Meta_reorderGoals(x_35, x_33, x_34, x_29, x_32, x_30); +lean_inc(x_31); +lean_inc_ref(x_30); +lean_inc(x_32); +lean_inc_ref(x_33); +x_39 = l___private_Lean_Meta_Tactic_Apply_0__Lean_Meta_reorderGoals(x_35, x_28, x_33, x_32, x_30, x_31); if (lean_obj_tag(x_39) == 0) { lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; @@ -5958,17 +5958,17 @@ x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); lean_dec_ref(x_39); x_41 = lean_array_get_size(x_38); -x_42 = lean_mk_empty_array_with_capacity(x_28); -x_43 = lean_nat_dec_lt(x_28, x_41); +x_42 = lean_mk_empty_array_with_capacity(x_29); +x_43 = lean_nat_dec_lt(x_29, x_41); if (x_43 == 0) { lean_dec(x_38); -x_11 = x_29; -x_12 = x_30; -x_13 = lean_box(0); -x_14 = x_32; +x_11 = x_30; +x_12 = x_31; +x_13 = x_32; +x_14 = x_33; x_15 = x_40; -x_16 = x_34; +x_16 = lean_box(0); x_17 = x_42; goto block_27; } @@ -5979,12 +5979,12 @@ x_44 = lean_nat_dec_le(x_41, x_41); if (x_44 == 0) { lean_dec(x_38); -x_11 = x_29; -x_12 = x_30; -x_13 = lean_box(0); -x_14 = x_32; +x_11 = x_30; +x_12 = x_31; +x_13 = x_32; +x_14 = x_33; x_15 = x_40; -x_16 = x_34; +x_16 = lean_box(0); x_17 = x_42; goto block_27; } @@ -5995,12 +5995,12 @@ x_45 = 0; x_46 = lean_usize_of_nat(x_41); x_47 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00Lean_MVarId_apply_spec__4(x_40, x_38, x_45, x_46, x_42); lean_dec(x_38); -x_11 = x_29; -x_12 = x_30; -x_13 = lean_box(0); -x_14 = x_32; +x_11 = x_30; +x_12 = x_31; +x_13 = x_32; +x_14 = x_33; x_15 = x_40; -x_16 = x_34; +x_16 = lean_box(0); x_17 = x_47; goto block_27; } @@ -6009,10 +6009,10 @@ goto block_27; else { lean_dec(x_38); -lean_dec_ref(x_34); -lean_dec_ref(x_32); -lean_dec(x_30); -lean_dec(x_29); +lean_dec_ref(x_33); +lean_dec(x_32); +lean_dec(x_31); +lean_dec_ref(x_30); return x_39; } } @@ -6020,10 +6020,10 @@ else { uint8_t x_48; lean_dec_ref(x_35); -lean_dec_ref(x_34); -lean_dec_ref(x_32); -lean_dec(x_30); -lean_dec(x_29); +lean_dec_ref(x_33); +lean_dec(x_32); +lean_dec(x_31); +lean_dec_ref(x_30); x_48 = !lean_is_exclusive(x_37); if (x_48 == 0) { diff --git a/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c index 767c8ec1d20a..cadb39c1f079 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c @@ -1769,7 +1769,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg(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) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_28; double x_29; double x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_39; double x_40; lean_object* x_41; double x_42; uint8_t x_43; lean_object* x_44; 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_64; double x_65; uint8_t x_66; lean_object* x_67; double x_68; lean_object* x_69; lean_object* x_70; lean_object* x_75; lean_object* x_76; uint8_t x_77; double x_78; lean_object* x_79; double x_80; lean_object* x_85; lean_object* x_86; lean_object* x_87; double x_88; double x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; uint8_t x_93; lean_object* x_127; double x_128; lean_object* x_129; double x_130; uint8_t x_131; lean_object* x_132; double x_133; lean_object* x_137; uint8_t x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_159; lean_object* x_160; double x_161; uint8_t x_162; lean_object* x_163; double x_164; uint8_t x_165; lean_object* x_199; lean_object* x_200; uint8_t x_201; double x_202; lean_object* x_203; double x_204; double x_205; lean_object* x_209; uint8_t x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; +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_28; uint8_t x_29; lean_object* x_30; double x_31; double x_32; lean_object* x_33; lean_object* x_34; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; double x_43; double x_44; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_64; lean_object* x_65; double x_66; lean_object* x_67; double x_68; lean_object* x_69; lean_object* x_70; uint8_t x_75; lean_object* x_76; lean_object* x_77; double x_78; lean_object* x_79; double x_80; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; double x_91; double x_92; uint8_t x_93; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; double x_131; double x_132; double x_133; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_159; lean_object* x_160; lean_object* x_161; double x_162; lean_object* x_163; double x_164; uint8_t x_165; uint8_t x_199; lean_object* x_200; lean_object* x_201; double x_202; lean_object* x_203; double x_204; double x_205; lean_object* x_209; uint8_t x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_249; x_11 = lean_ctor_get(x_8, 2); x_12 = lean_ctor_get(x_8, 5); lean_inc(x_1); @@ -1807,7 +1807,7 @@ goto block_248; block_27: { lean_object* x_22; -x_22 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__4(x_13, x_16, x_12, x_14, x_17, x_18, x_19, x_20); +x_22 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__4(x_15, x_16, x_12, x_14, x_17, x_18, x_19, x_20); lean_dec(x_20); lean_dec(x_18); lean_dec_ref(x_17); @@ -1815,13 +1815,13 @@ if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_dec_ref(x_22); -x_23 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_15); +x_23 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_13); return x_23; } else { uint8_t x_24; -lean_dec_ref(x_15); +lean_dec_ref(x_13); x_24 = !lean_is_exclusive(x_22); if (x_24 == 0) { @@ -1841,7 +1841,7 @@ return x_26; } block_38: { -if (x_32 == 0) +if (x_29 == 0) { double x_35; lean_object* x_36; x_35 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__0; @@ -1853,7 +1853,7 @@ lean_ctor_set_float(x_36, sizeof(void*)*2 + 8, x_35); lean_ctor_set_uint8(x_36, sizeof(void*)*2 + 16, x_4); x_13 = x_28; x_14 = x_33; -x_15 = x_31; +x_15 = x_30; x_16 = x_36; x_17 = x_6; x_18 = x_7; @@ -1868,12 +1868,12 @@ lean_object* x_37; x_37 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_37, 0, x_1); lean_ctor_set(x_37, 1, x_5); -lean_ctor_set_float(x_37, sizeof(void*)*2, x_29); -lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_30); +lean_ctor_set_float(x_37, sizeof(void*)*2, x_32); +lean_ctor_set_float(x_37, sizeof(void*)*2 + 8, x_31); lean_ctor_set_uint8(x_37, sizeof(void*)*2 + 16, x_4); x_13 = x_28; x_14 = x_33; -x_15 = x_31; +x_15 = x_30; x_16 = x_37; x_17 = x_6; x_18 = x_7; @@ -1890,8 +1890,8 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_41); -x_45 = lean_apply_6(x_2, x_41, x_6, x_7, x_8, x_9, lean_box(0)); +lean_inc_ref(x_39); +x_45 = lean_apply_6(x_2, x_39, x_6, x_7, x_8, x_9, lean_box(0)); if (lean_obj_tag(x_45) == 0) { lean_object* x_46; @@ -1901,8 +1901,8 @@ lean_dec_ref(x_45); x_28 = x_39; x_29 = x_40; x_30 = x_42; -x_31 = x_41; -x_32 = x_43; +x_31 = x_43; +x_32 = x_44; x_33 = x_46; x_34 = lean_box(0); goto block_38; @@ -1915,8 +1915,8 @@ x_47 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lea x_28 = x_39; x_29 = x_40; x_30 = x_42; -x_31 = x_41; -x_32 = x_43; +x_31 = x_43; +x_32 = x_44; x_33 = x_47; x_34 = lean_box(0); goto block_38; @@ -1925,7 +1925,7 @@ goto block_38; block_63: { lean_object* x_58; -x_58 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__4(x_50, x_52, x_12, x_49, x_53, x_54, x_55, x_56); +x_58 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__4(x_50, x_52, x_12, x_51, x_53, x_54, x_55, x_56); lean_dec(x_56); lean_dec(x_54); lean_dec_ref(x_53); @@ -1933,13 +1933,13 @@ if (lean_obj_tag(x_58) == 0) { lean_object* x_59; lean_dec_ref(x_58); -x_59 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_51); +x_59 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_49); return x_59; } else { uint8_t x_60; -lean_dec_ref(x_51); +lean_dec_ref(x_49); x_60 = !lean_is_exclusive(x_58); if (x_60 == 0) { @@ -1959,7 +1959,7 @@ return x_62; } block_74: { -if (x_66 == 0) +if (x_64 == 0) { double x_71; lean_object* x_72; x_71 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__0; @@ -1969,9 +1969,9 @@ lean_ctor_set(x_72, 1, x_5); lean_ctor_set_float(x_72, sizeof(void*)*2, x_71); lean_ctor_set_float(x_72, sizeof(void*)*2 + 8, x_71); lean_ctor_set_uint8(x_72, sizeof(void*)*2 + 16, x_4); -x_49 = x_69; -x_50 = x_64; -x_51 = x_67; +x_49 = x_65; +x_50 = x_67; +x_51 = x_69; x_52 = x_72; x_53 = x_6; x_54 = x_7; @@ -1987,11 +1987,11 @@ x_73 = lean_alloc_ctor(0, 2, 17); lean_ctor_set(x_73, 0, x_1); lean_ctor_set(x_73, 1, x_5); lean_ctor_set_float(x_73, sizeof(void*)*2, x_68); -lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_65); +lean_ctor_set_float(x_73, sizeof(void*)*2 + 8, x_66); lean_ctor_set_uint8(x_73, sizeof(void*)*2 + 16, x_4); -x_49 = x_69; -x_50 = x_64; -x_51 = x_67; +x_49 = x_65; +x_50 = x_67; +x_51 = x_69; x_52 = x_73; x_53 = x_6; x_54 = x_7; @@ -2008,8 +2008,8 @@ lean_inc(x_9); lean_inc_ref(x_8); lean_inc(x_7); lean_inc_ref(x_6); -lean_inc_ref(x_79); -x_81 = lean_apply_6(x_2, x_79, x_6, x_7, x_8, x_9, lean_box(0)); +lean_inc_ref(x_76); +x_81 = lean_apply_6(x_2, x_76, x_6, x_7, x_8, x_9, lean_box(0)); if (lean_obj_tag(x_81) == 0) { lean_object* x_82; @@ -2017,8 +2017,8 @@ x_82 = lean_ctor_get(x_81, 0); lean_inc(x_82); lean_dec_ref(x_81); x_64 = x_75; -x_65 = x_78; -x_66 = x_77; +x_65 = x_76; +x_66 = x_78; x_67 = x_79; x_68 = x_80; x_69 = x_82; @@ -2031,8 +2031,8 @@ lean_object* x_83; lean_dec_ref(x_81); x_83 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__2; x_64 = x_75; -x_65 = x_78; -x_66 = x_77; +x_65 = x_76; +x_66 = x_78; x_67 = x_79; x_68 = x_80; x_69 = x_83; @@ -2068,12 +2068,12 @@ if (x_98 == 0) { lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; x_99 = lean_ctor_get(x_97, 0); -x_100 = l_Lean_PersistentArray_append___redArg(x_87, x_99); +x_100 = l_Lean_PersistentArray_append___redArg(x_90, x_99); lean_dec_ref(x_99); lean_ctor_set(x_97, 0, x_100); x_101 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_90); +x_102 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_87); return x_102; } else @@ -2083,7 +2083,7 @@ x_103 = lean_ctor_get_uint64(x_97, sizeof(void*)*1); x_104 = lean_ctor_get(x_97, 0); lean_inc(x_104); lean_dec(x_97); -x_105 = l_Lean_PersistentArray_append___redArg(x_87, x_104); +x_105 = l_Lean_PersistentArray_append___redArg(x_90, x_104); lean_dec_ref(x_104); x_106 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_106, 0, x_105); @@ -2091,7 +2091,7 @@ lean_ctor_set_uint64(x_106, sizeof(void*)*1, x_103); lean_ctor_set(x_95, 4, x_106); x_107 = lean_st_ref_set(x_9, x_95); lean_dec(x_9); -x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_90); +x_108 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_87); return x_108; } } @@ -2127,7 +2127,7 @@ if (lean_is_exclusive(x_109)) { lean_dec_ref(x_109); x_120 = lean_box(0); } -x_121 = l_Lean_PersistentArray_append___redArg(x_87, x_119); +x_121 = l_Lean_PersistentArray_append___redArg(x_90, x_119); lean_dec_ref(x_119); if (lean_is_scalar(x_120)) { x_122 = lean_alloc_ctor(0, 1, 8); @@ -2148,7 +2148,7 @@ lean_ctor_set(x_123, 7, x_116); lean_ctor_set(x_123, 8, x_117); x_124 = lean_st_ref_set(x_9, x_123); lean_dec(x_9); -x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_90); +x_125 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_87); return x_125; } } @@ -2156,10 +2156,10 @@ else { x_39 = x_87; x_40 = x_88; -x_41 = x_90; -x_42 = x_89; +x_41 = lean_box(0); +x_42 = x_90; x_43 = x_91; -x_44 = lean_box(0); +x_44 = x_92; goto block_48; } } @@ -2167,24 +2167,24 @@ else { x_39 = x_87; x_40 = x_88; -x_41 = x_90; -x_42 = x_89; +x_41 = lean_box(0); +x_42 = x_90; x_43 = x_91; -x_44 = lean_box(0); +x_44 = x_92; goto block_48; } } block_136: { double x_134; uint8_t x_135; -x_134 = lean_float_sub(x_130, x_128); +x_134 = lean_float_sub(x_131, x_132); x_135 = lean_float_decLt(x_133, x_134); x_87 = x_127; x_88 = x_128; -x_89 = x_130; -x_90 = x_129; +x_89 = lean_box(0); +x_90 = x_130; x_91 = x_131; -x_92 = lean_box(0); +x_92 = x_132; x_93 = x_135; goto block_126; } @@ -2201,18 +2201,18 @@ x_148 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Le x_149 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__3(x_11, x_148); if (x_149 == 0) { -x_87 = x_137; -x_88 = x_145; -x_89 = x_147; -x_90 = x_140; -x_91 = x_149; -x_92 = lean_box(0); +x_87 = x_140; +x_88 = x_149; +x_89 = lean_box(0); +x_90 = x_138; +x_91 = x_147; +x_92 = x_145; x_93 = x_149; goto block_126; } else { -if (x_138 == 0) +if (x_137 == 0) { lean_object* x_150; lean_object* x_151; double x_152; double x_153; double x_154; x_150 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__5; @@ -2220,12 +2220,12 @@ x_151 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Me x_152 = lean_float_of_nat(x_151); x_153 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__6; x_154 = lean_float_div(x_152, x_153); -x_127 = x_137; -x_128 = x_145; -x_129 = x_140; -x_130 = x_147; -x_131 = x_149; -x_132 = lean_box(0); +x_127 = x_140; +x_128 = x_149; +x_129 = lean_box(0); +x_130 = x_138; +x_131 = x_147; +x_132 = x_145; x_133 = x_154; goto block_136; } @@ -2235,12 +2235,12 @@ lean_object* x_155; lean_object* x_156; double x_157; x_155 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__5; x_156 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__6(x_11, x_155); x_157 = lean_float_of_nat(x_156); -x_127 = x_137; -x_128 = x_145; -x_129 = x_140; -x_130 = x_147; -x_131 = x_149; -x_132 = lean_box(0); +x_127 = x_140; +x_128 = x_149; +x_129 = lean_box(0); +x_130 = x_138; +x_131 = x_147; +x_132 = x_145; x_133 = x_157; goto block_136; } @@ -2274,12 +2274,12 @@ if (x_170 == 0) { lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; x_171 = lean_ctor_get(x_169, 0); -x_172 = l_Lean_PersistentArray_append___redArg(x_159, x_171); +x_172 = l_Lean_PersistentArray_append___redArg(x_163, x_171); lean_dec_ref(x_171); lean_ctor_set(x_169, 0, x_172); x_173 = lean_st_ref_set(x_9, x_167); lean_dec(x_9); -x_174 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_163); +x_174 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_160); return x_174; } else @@ -2289,7 +2289,7 @@ x_175 = lean_ctor_get_uint64(x_169, sizeof(void*)*1); x_176 = lean_ctor_get(x_169, 0); lean_inc(x_176); lean_dec(x_169); -x_177 = l_Lean_PersistentArray_append___redArg(x_159, x_176); +x_177 = l_Lean_PersistentArray_append___redArg(x_163, x_176); lean_dec_ref(x_176); x_178 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_178, 0, x_177); @@ -2297,7 +2297,7 @@ lean_ctor_set_uint64(x_178, sizeof(void*)*1, x_175); lean_ctor_set(x_167, 4, x_178); x_179 = lean_st_ref_set(x_9, x_167); lean_dec(x_9); -x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_163); +x_180 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_160); return x_180; } } @@ -2333,7 +2333,7 @@ if (lean_is_exclusive(x_181)) { lean_dec_ref(x_181); x_192 = lean_box(0); } -x_193 = l_Lean_PersistentArray_append___redArg(x_159, x_191); +x_193 = l_Lean_PersistentArray_append___redArg(x_163, x_191); lean_dec_ref(x_191); if (lean_is_scalar(x_192)) { x_194 = lean_alloc_ctor(0, 1, 8); @@ -2354,16 +2354,16 @@ lean_ctor_set(x_195, 7, x_188); lean_ctor_set(x_195, 8, x_189); x_196 = lean_st_ref_set(x_9, x_195); lean_dec(x_9); -x_197 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_163); +x_197 = l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__5___redArg(x_160); return x_197; } } else { x_75 = x_159; -x_76 = lean_box(0); -x_77 = x_162; -x_78 = x_161; +x_76 = x_160; +x_77 = lean_box(0); +x_78 = x_162; x_79 = x_163; x_80 = x_164; goto block_84; @@ -2372,9 +2372,9 @@ goto block_84; else { x_75 = x_159; -x_76 = lean_box(0); -x_77 = x_162; -x_78 = x_161; +x_76 = x_160; +x_77 = lean_box(0); +x_78 = x_162; x_79 = x_163; x_80 = x_164; goto block_84; @@ -2386,9 +2386,9 @@ double x_206; uint8_t x_207; x_206 = lean_float_sub(x_202, x_204); x_207 = lean_float_decLt(x_205, x_206); x_159 = x_199; -x_160 = lean_box(0); -x_161 = x_202; -x_162 = x_201; +x_160 = x_200; +x_161 = lean_box(0); +x_162 = x_202; x_163 = x_203; x_164 = x_204; x_165 = x_207; @@ -2398,17 +2398,17 @@ goto block_198; { lean_object* x_214; double x_215; double x_216; lean_object* x_217; uint8_t x_218; x_214 = lean_io_get_num_heartbeats(); -x_215 = lean_float_of_nat(x_211); +x_215 = lean_float_of_nat(x_209); x_216 = lean_float_of_nat(x_214); x_217 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__4; x_218 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__3(x_11, x_217); if (x_218 == 0) { -x_159 = x_209; -x_160 = lean_box(0); -x_161 = x_216; -x_162 = x_218; -x_163 = x_212; +x_159 = x_218; +x_160 = x_212; +x_161 = lean_box(0); +x_162 = x_216; +x_163 = x_211; x_164 = x_215; x_165 = x_218; goto block_198; @@ -2423,11 +2423,11 @@ x_220 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Me x_221 = lean_float_of_nat(x_220); x_222 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__6; x_223 = lean_float_div(x_221, x_222); -x_199 = x_209; -x_200 = lean_box(0); -x_201 = x_218; +x_199 = x_218; +x_200 = x_212; +x_201 = lean_box(0); x_202 = x_216; -x_203 = x_212; +x_203 = x_211; x_204 = x_215; x_205 = x_223; goto block_208; @@ -2438,11 +2438,11 @@ lean_object* x_224; lean_object* x_225; double x_226; x_224 = l_Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1___redArg___closed__5; x_225 = l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run_spec__1_spec__6(x_11, x_224); x_226 = lean_float_of_nat(x_225); -x_199 = x_209; -x_200 = lean_box(0); -x_201 = x_218; +x_199 = x_218; +x_200 = x_212; +x_201 = lean_box(0); x_202 = x_216; -x_203 = x_212; +x_203 = x_211; x_204 = x_215; x_205 = x_226; goto block_208; @@ -2474,8 +2474,8 @@ x_234 = !lean_is_exclusive(x_233); if (x_234 == 0) { lean_ctor_set_tag(x_233, 1); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_233; x_141 = lean_box(0); @@ -2489,8 +2489,8 @@ lean_inc(x_235); lean_dec(x_233); x_236 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_236, 0, x_235); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_236; x_141 = lean_box(0); @@ -2504,8 +2504,8 @@ x_237 = !lean_is_exclusive(x_233); if (x_237 == 0) { lean_ctor_set_tag(x_233, 0); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_233; x_141 = lean_box(0); @@ -2519,8 +2519,8 @@ lean_inc(x_238); lean_dec(x_233); x_239 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_239, 0, x_238); -x_137 = x_229; -x_138 = x_231; +x_137 = x_231; +x_138 = x_229; x_139 = x_232; x_140 = x_239; x_141 = lean_box(0); @@ -2544,9 +2544,9 @@ x_242 = !lean_is_exclusive(x_241); if (x_242 == 0) { lean_ctor_set_tag(x_241, 1); -x_209 = x_229; +x_209 = x_240; x_210 = x_231; -x_211 = x_240; +x_211 = x_229; x_212 = x_241; x_213 = lean_box(0); goto block_227; @@ -2559,9 +2559,9 @@ lean_inc(x_243); lean_dec(x_241); x_244 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_244, 0, x_243); -x_209 = x_229; +x_209 = x_240; x_210 = x_231; -x_211 = x_240; +x_211 = x_229; x_212 = x_244; x_213 = lean_box(0); goto block_227; @@ -2574,9 +2574,9 @@ x_245 = !lean_is_exclusive(x_241); if (x_245 == 0) { lean_ctor_set_tag(x_241, 0); -x_209 = x_229; +x_209 = x_240; x_210 = x_231; -x_211 = x_240; +x_211 = x_229; x_212 = x_241; x_213 = lean_box(0); goto block_227; @@ -2589,9 +2589,9 @@ lean_inc(x_246); lean_dec(x_241); x_247 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_247, 0, x_246); -x_209 = x_229; +x_209 = x_240; x_210 = x_231; -x_211 = x_240; +x_211 = x_229; x_212 = x_247; x_213 = lean_box(0); goto block_227; @@ -5273,11 +5273,11 @@ return x_22; if (x_28 == 0) { lean_object* x_29; -lean_dec_ref(x_26); -x_29 = l_Lean_Meta_SavedState_restore___redArg(x_25, x_12, x_14); +lean_dec_ref(x_25); +x_29 = l_Lean_Meta_SavedState_restore___redArg(x_26, x_12, x_14); lean_dec(x_14); lean_dec(x_12); -lean_dec_ref(x_25); +lean_dec_ref(x_26); if (lean_obj_tag(x_29) == 0) { lean_dec_ref(x_29); @@ -5310,11 +5310,11 @@ return x_32; } else { -lean_dec_ref(x_25); +lean_dec_ref(x_26); lean_dec(x_14); lean_dec(x_12); lean_dec(x_3); -x_22 = x_26; +x_22 = x_25; goto block_24; } } @@ -5409,8 +5409,8 @@ if (x_53 == 0) { uint8_t x_54; x_54 = l_Lean_Exception_isRuntime(x_52); -x_25 = x_50; -x_26 = x_51; +x_25 = x_51; +x_26 = x_50; x_27 = lean_box(0); x_28 = x_54; goto block_33; @@ -5418,8 +5418,8 @@ goto block_33; else { lean_dec(x_52); -x_25 = x_50; -x_26 = x_51; +x_25 = x_51; +x_26 = x_50; x_27 = lean_box(0); x_28 = x_53; goto block_33; diff --git a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c index 902954c743d5..287a9b5755ac 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c +++ b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c @@ -110,7 +110,6 @@ static lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknow LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__21___redArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstVal___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__3_spec__5_spec__11___redArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase___lam__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__5___lam__3(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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_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*); @@ -265,6 +264,7 @@ static lean_object* l_panic___at___00Lean_Meta_MatcherApp_transform___at___00__p LEAN_EXPORT lean_object* l_Lean_getConstVal___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknownIdentifierMessage___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__2_spec__8_spec__33_spec__42_spec__46_spec__48___redArg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__28___closed__4; LEAN_EXPORT uint8_t l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__25_spec__27_spec__41___lam__0(uint8_t, uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__5(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -374,6 +374,7 @@ lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__28___closed__16; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___closed__1; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__initFn___closed__8_00___x40_Lean_Meta_Tactic_FunInd_922168289____hygCtx___hyg_2_; +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__17___closed__4; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_initFn___lam__0___closed__0_00___x40_Lean_Meta_Tactic_FunInd_4256658486____hygCtx___hyg_2_; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__28___closed__29; @@ -609,7 +610,6 @@ static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_de LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_projectMutualInduct_spec__1___lam__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_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__4_spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_isFunInductName___closed__1; -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_M_run___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6_spec__9___redArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_M_branch___redArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -656,9 +656,9 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_ lean_object* l_Lean_Meta_isTypeCorrect(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___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveCases___lam__0(lean_object*); +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0; LEAN_EXPORT lean_object* l_Lean_Elab_FixedParamPerm_forallTelescope___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__20___redArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_initFn___lam__0_00___x40_Lean_Meta_Tactic_FunInd_4256658486____hygCtx___hyg_2_(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__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_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__15(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -785,7 +785,6 @@ static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_de static lean_object* l_Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12___closed__12; LEAN_EXPORT lean_object* l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_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_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_M_localMapM___redArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___boxed(lean_object**); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); static lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknownIdentifierMessage___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__2_spec__8_spec__33_spec__42_spec__46_spec__48___redArg___closed__12; lean_object* l_Lean_Meta_Match_MatcherInfo_getMotivePos(lean_object*); @@ -806,6 +805,7 @@ lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lea lean_object* l_Array_empty(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__4___closed__8; LEAN_EXPORT lean_object* l_Lean_logAt___at___00Lean_log___at___00Lean_logError___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__25_spec__27_spec__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__21(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_unpackMutualInduction_doRealize_spec__0___lam__0___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__10___lam__0___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -823,6 +823,7 @@ LEAN_EXPORT lean_object* l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__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*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__28___closed__25; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__initFn___closed__15_00___x40_Lean_Meta_Tactic_FunInd_922168289____hygCtx___hyg_2_; +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__4___lam__0___boxed(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*); @@ -880,7 +881,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_withUserNames___at___00Lean_Meta static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__0; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__4_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* l_Lean_MessageData_ofFormat(lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2; static lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknownIdentifierMessage___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__2_spec__8_spec__33_spec__42_spec__46_spec__48___redArg___closed__20; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_refinedArguments_spec__1___redArg(uint8_t, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_PersistentArray_forIn___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f_spec__1_spec__2_spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1034,6 +1034,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunI LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Meta_withLocalDeclsDND___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_abstractIndependentMVars_spec__6_spec__8(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_unpackMutualInduction_doRealize___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_withUserNames___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__5_spec__14___redArg___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_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1; lean_object* l_Lean_Expr_constName_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstVal___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__3_spec__5_spec__11_spec__14___redArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__10___closed__5; @@ -1302,7 +1303,6 @@ LEAN_EXPORT lean_object* l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_ static lean_object* l_Lean_Expr_withAppAux___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_unpackMutualInduction_doRealize_spec__0___closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0_spec__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__4___lam__0(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__8___closed__7; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_abstractIndependentMVars_spec__4___redArg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__17___closed__0; @@ -1338,7 +1338,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunI static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__20___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_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___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__2; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0(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*); static lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknownIdentifierMessage___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__2_spec__8_spec__33_spec__42_spec__46_spec__48___redArg___closed__0; LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_WellFounded_opaqueFix_u2083___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__5_spec__19___redArg___lam__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*); @@ -1355,7 +1354,6 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___00Lean_throwUnknownIdentifie static lean_object* l_Lean_Expr_withAppAux___at___00Lean_Expr_withAppAux___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanPackedArgs_spec__0_spec__0___closed__4; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__21___closed__0; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00Lean_PersistentArray_forInAux___at___00Lean_PersistentArray_forIn___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f_spec__1_spec__1_spec__3_spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__4___closed__5; lean_object* l_Lean_Meta_MatcherApp_inferMatchType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1370,6 +1368,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___00__private_Lean_Meta_Ta LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__5___redArg(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_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deduplicateIHs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanupAfter_allHeqToEq_spec__0___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3; LEAN_EXPORT lean_object* l_Lean_mkUnknownIdentifierMessageCore___at___00Lean_mkUnknownIdentifierMessage___at___00Lean_throwUnknownIdentifierAt___at___00Lean_throwUnknownConstantAt___at___00Lean_throwUnknownConstant___at___00Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__4_spec__4_spec__7_spec__18_spec__28_spec__31_spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_forallAltTelescope_x27___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__5_spec__18___redArg___lam__0(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_heqToEq(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1403,7 +1402,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___00__private_Lean_Met static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_withLetDecls___redArg___closed__0; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__19(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__27___closed__4; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2(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_EXPORT lean_object* l_WellFounded_opaqueFix_u2083___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__24___redArg___lam__0(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___00Lean_Meta_matchMatcherApp_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__1_spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_unpackMutualInduction_doRealize___lam__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*); @@ -1416,7 +1414,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at extern lean_object* l_Lean_Elab_Structural_instInhabitedEqnInfo_default; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___00Lean_getConstVal___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__3_spec__5___redArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___00Lean_Meta_withLocalDeclsDND___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_abstractIndependentMVars_spec__6_spec__9(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect___lam__4___closed__0; static lean_object* l_Lean_Expr_withAppAux___at___00Lean_Expr_withAppAux___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanPackedArgs_spec__0_spec__0___closed__2; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__3; @@ -1490,7 +1487,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunI LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___00Lean_Expr_withAppAux___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanPackedArgs_spec__0_spec__0___closed__12; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Meta_Transform_0__Lean_Meta_transformWithCache_visit___at___00Lean_Meta_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_cleanPackedArgs_spec__1_spec__2_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___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_withLetDecls_go_spec__0___redArg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_abstractIndependentMVars_spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_WellFounded_opaqueFix_u2083___at___00Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12_spec__29___redArg___closed__0; @@ -1619,7 +1615,6 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__8___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg(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_FunInd_0__Lean_Tactic_FunInd_setNaryFunIndInfo___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_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed(lean_object**); static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase___lam__1___closed__1; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__13_spec__36(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1668,6 +1663,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunI LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___00Std_DHashMap_Internal_Raw_u2080_insert___at___00__private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0_spec__6_spec__9___redArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__9___redArg___lam__1(uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Option_get___at___00Lean_withTraceNode___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__13_spec__37(lean_object*, lean_object*); +static lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; static lean_object* l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__28___closed__10; static lean_object* l_Lean_Meta_MatcherApp_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__12___closed__9; LEAN_EXPORT lean_object* l_panic___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_withLetDecls_spec__0___redArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -95511,8 +95507,8 @@ return x_10; block_24: { lean_object* x_23; -lean_dec(x_19); -x_23 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6_spec__11___redArg(x_21, x_20, x_22); +lean_dec(x_21); +x_23 = l___private_Init_Data_Array_QSort_Basic_0__Array_qsort_sort___at___00Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6_spec__11___redArg(x_20, x_19, x_22); lean_dec(x_22); x_13 = x_23; goto block_18; @@ -95520,23 +95516,23 @@ goto block_18; block_30: { uint8_t x_29; -x_29 = lean_nat_dec_le(x_28, x_26); +x_29 = lean_nat_dec_le(x_28, x_25); if (x_29 == 0) { -lean_dec(x_26); +lean_dec(x_25); lean_inc(x_28); -x_19 = x_25; -x_20 = x_28; +x_19 = x_28; +x_20 = x_26; x_21 = x_27; x_22 = x_28; goto block_24; } else { -x_19 = x_25; -x_20 = x_28; +x_19 = x_28; +x_20 = x_26; x_21 = x_27; -x_22 = x_26; +x_22 = x_25; goto block_24; } } @@ -95555,17 +95551,17 @@ x_37 = lean_nat_dec_le(x_33, x_36); if (x_37 == 0) { lean_inc(x_36); -x_25 = x_32; -x_26 = x_36; -x_27 = x_31; +x_25 = x_36; +x_26 = x_31; +x_27 = x_32; x_28 = x_36; goto block_30; } else { -x_25 = x_32; -x_26 = x_36; -x_27 = x_31; +x_25 = x_36; +x_26 = x_31; +x_27 = x_32; x_28 = x_33; goto block_30; } @@ -96643,1363 +96639,215 @@ return x_4; } LEAN_EXPORT lean_object* l_Array_idxOf_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__11(lean_object* x_1, lean_object* x_2) { _start: -{ -lean_object* x_3; -x_3 = l_Array_finIdxOf_x3f___at___00Array_idxOf_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__11_spec__18(x_1, x_2); -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_4; -x_4 = lean_box(0); -return x_4; -} -else -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -return x_3; -} -else -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_ctor_get(x_3, 0); -lean_inc(x_6); -lean_dec(x_3); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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, uint8_t x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Expr_getAppFn(x_9); -x_11 = l_Array_idxOf_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__11(x_1, x_10); -lean_dec_ref(x_10); -if (lean_obj_tag(x_11) == 1) -{ -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_11, 0); -lean_inc(x_12); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - x_13 = x_11; -} else { - lean_dec_ref(x_11); - x_13 = lean_box(0); -} -x_14 = l_Lean_Expr_getAppNumArgs(x_9); -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_array_get_borrowed(x_15, x_2, x_12); -x_17 = lean_nat_dec_eq(x_14, x_16); -if (x_17 == 0) -{ -lean_object* x_18; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec_ref(x_9); -lean_dec_ref(x_5); -lean_dec_ref(x_3); -x_18 = lean_box(0); -return x_18; -} -else -{ -lean_object* x_19; lean_object* x_20; -x_19 = lean_array_get_borrowed(x_3, x_4, x_12); -if (x_8 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_32 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0___lam__1___closed__0; -lean_inc(x_14); -x_33 = lean_mk_array(x_14, x_32); -x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_nat_sub(x_14, x_34); -lean_dec(x_14); -x_36 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_33, x_35); -x_20 = x_36; -goto block_31; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_37 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0___lam__1___closed__0; -lean_inc(x_14); -x_38 = lean_mk_array(x_14, x_37); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_sub(x_14, x_39); -lean_dec(x_14); -x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_38, x_40); -x_42 = lean_array_pop(x_41); -x_20 = x_42; -goto block_31; -} -block_31: -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_ctor_get(x_21, 0); -x_23 = lean_ctor_get(x_21, 1); -x_24 = lean_array_get_borrowed(x_5, x_6, x_12); -lean_dec(x_12); -lean_inc(x_24); -x_25 = l_Lean_Elab_FixedParamPerm_buildArgs___redArg(x_24, x_7, x_20); -x_26 = lean_box(0); -lean_inc(x_23); -x_27 = l_List_mapTR_loop___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__4(x_23, x_26); -lean_inc(x_22); -x_28 = l_Lean_Expr_const___override(x_22, x_27); -x_29 = l_Lean_mkAppN(x_28, x_25); -lean_dec_ref(x_25); -if (lean_is_scalar(x_13)) { - x_30 = lean_alloc_ctor(1, 1, 0); -} else { - x_30 = x_13; -} -lean_ctor_set(x_30, 0, x_29); -return x_30; -} -} -} -else -{ -lean_object* x_43; -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec_ref(x_5); -lean_dec_ref(x_3); -x_43 = lean_box(0); -return x_43; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_8); -x_11 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_10, x_9); -lean_dec_ref(x_7); -lean_dec_ref(x_6); -lean_dec_ref(x_4); -lean_dec_ref(x_2); -lean_dec_ref(x_1); -return x_11; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = l_Lean_Expr_fvarId_x21(x_1); -x_15 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__13___closed__2; -lean_inc(x_2); -x_16 = lean_array_push(x_15, x_2); -lean_inc(x_14); -x_17 = lean_array_push(x_16, x_14); -x_18 = lean_mk_empty_array_with_capacity(x_3); -x_19 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody(x_17, x_18, x_6, x_2, x_14, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12); -return x_19; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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_ref(x_1); -return x_14; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("replacing ", 10, 10); -return x_1; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" with ", 6, 6); -return x_1; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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_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_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_130; -lean_inc(x_1); -x_130 = l_Lean_isTracingEnabledFor___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase_spec__1___redArg(x_1, x_12, x_13, x_16); -if (lean_obj_tag(x_130) == 0) -{ -lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -lean_dec_ref(x_130); -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_132, 0); -x_134 = lean_unbox(x_133); -if (x_134 == 0) -{ -lean_object* x_135; lean_object* x_136; -lean_dec(x_1); -x_135 = lean_ctor_get(x_131, 1); -lean_inc(x_135); -lean_dec(x_131); -x_136 = lean_ctor_get(x_132, 1); -lean_inc(x_136); -lean_dec(x_132); -x_49 = x_136; -x_50 = x_135; -x_51 = x_14; -x_52 = x_15; -x_53 = x_16; -x_54 = x_17; -x_55 = lean_box(0); -goto block_129; -} -else -{ -uint8_t x_137; -x_137 = !lean_is_exclusive(x_131); -if (x_137 == 0) -{ -lean_object* x_138; lean_object* x_139; uint8_t x_140; -x_138 = lean_ctor_get(x_131, 1); -x_139 = lean_ctor_get(x_131, 0); -lean_dec(x_139); -x_140 = !lean_is_exclusive(x_132); -if (x_140 == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_141 = lean_ctor_get(x_132, 1); -x_142 = lean_ctor_get(x_132, 0); -lean_dec(x_142); -x_143 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; -lean_inc(x_10); -x_144 = l_Lean_Expr_fvar___override(x_10); -x_145 = l_Lean_MessageData_ofExpr(x_144); -lean_ctor_set_tag(x_132, 7); -lean_ctor_set(x_132, 1, x_145); -lean_ctor_set(x_132, 0, x_143); -x_146 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; -lean_ctor_set_tag(x_131, 7); -lean_ctor_set(x_131, 1, x_146); -lean_inc_ref(x_4); -x_147 = l_Lean_MessageData_ofExpr(x_4); -x_148 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_148, 0, x_131); -lean_ctor_set(x_148, 1, x_147); -x_149 = l_Lean_addTrace___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase_spec__2(x_1, x_148, x_141, x_138, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_149) == 0) -{ -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -lean_dec_ref(x_149); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_150, 1); -lean_inc(x_152); -lean_dec(x_150); -x_153 = lean_ctor_get(x_151, 1); -lean_inc(x_153); -lean_dec(x_151); -x_49 = x_153; -x_50 = x_152; -x_51 = x_14; -x_52 = x_15; -x_53 = x_16; -x_54 = x_17; -x_55 = lean_box(0); -goto block_129; -} -else -{ -uint8_t x_154; -lean_dec(x_17); -lean_dec_ref(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); -lean_dec_ref(x_11); -lean_dec(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_8); -lean_dec_ref(x_7); -lean_dec(x_6); -lean_dec_ref(x_5); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_154 = !lean_is_exclusive(x_149); -if (x_154 == 0) -{ -return x_149; -} -else -{ -lean_object* x_155; lean_object* x_156; -x_155 = lean_ctor_get(x_149, 0); -lean_inc(x_155); -lean_dec(x_149); -x_156 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_156, 0, x_155); -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; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_157 = lean_ctor_get(x_132, 1); -lean_inc(x_157); -lean_dec(x_132); -x_158 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; -lean_inc(x_10); -x_159 = l_Lean_Expr_fvar___override(x_10); -x_160 = l_Lean_MessageData_ofExpr(x_159); -x_161 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_161, 0, x_158); -lean_ctor_set(x_161, 1, x_160); -x_162 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; -lean_ctor_set_tag(x_131, 7); -lean_ctor_set(x_131, 1, x_162); -lean_ctor_set(x_131, 0, x_161); -lean_inc_ref(x_4); -x_163 = l_Lean_MessageData_ofExpr(x_4); -x_164 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_164, 0, x_131); -lean_ctor_set(x_164, 1, x_163); -x_165 = l_Lean_addTrace___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase_spec__2(x_1, x_164, x_157, x_138, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_165) == 0) -{ -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -lean_dec_ref(x_165); -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 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -lean_dec(x_167); -x_49 = x_169; -x_50 = x_168; -x_51 = x_14; -x_52 = x_15; -x_53 = x_16; -x_54 = x_17; -x_55 = lean_box(0); -goto block_129; -} -else -{ -lean_object* x_170; lean_object* x_171; lean_object* x_172; -lean_dec(x_17); -lean_dec_ref(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); -lean_dec_ref(x_11); -lean_dec(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_8); -lean_dec_ref(x_7); -lean_dec(x_6); -lean_dec_ref(x_5); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_170 = lean_ctor_get(x_165, 0); -lean_inc(x_170); -if (lean_is_exclusive(x_165)) { - lean_ctor_release(x_165, 0); - x_171 = x_165; -} else { - lean_dec_ref(x_165); - x_171 = lean_box(0); -} -if (lean_is_scalar(x_171)) { - x_172 = lean_alloc_ctor(1, 1, 0); -} else { - x_172 = x_171; -} -lean_ctor_set(x_172, 0, x_170); -return x_172; -} -} -} -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; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_173 = lean_ctor_get(x_131, 1); -lean_inc(x_173); -lean_dec(x_131); -x_174 = lean_ctor_get(x_132, 1); -lean_inc(x_174); -if (lean_is_exclusive(x_132)) { - lean_ctor_release(x_132, 0); - lean_ctor_release(x_132, 1); - x_175 = x_132; -} else { - lean_dec_ref(x_132); - x_175 = lean_box(0); -} -x_176 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; -lean_inc(x_10); -x_177 = l_Lean_Expr_fvar___override(x_10); -x_178 = l_Lean_MessageData_ofExpr(x_177); -if (lean_is_scalar(x_175)) { - x_179 = lean_alloc_ctor(7, 2, 0); -} else { - x_179 = x_175; - lean_ctor_set_tag(x_179, 7); -} -lean_ctor_set(x_179, 0, x_176); -lean_ctor_set(x_179, 1, x_178); -x_180 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; -x_181 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_181, 0, x_179); -lean_ctor_set(x_181, 1, x_180); -lean_inc_ref(x_4); -x_182 = l_Lean_MessageData_ofExpr(x_4); -x_183 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -x_184 = l_Lean_addTrace___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionCase_spec__2(x_1, x_183, x_174, x_173, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_184) == 0) -{ -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_185 = lean_ctor_get(x_184, 0); -lean_inc(x_185); -lean_dec_ref(x_184); -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_188 = lean_ctor_get(x_186, 1); -lean_inc(x_188); -lean_dec(x_186); -x_49 = x_188; -x_50 = x_187; -x_51 = x_14; -x_52 = x_15; -x_53 = x_16; -x_54 = x_17; -x_55 = lean_box(0); -goto block_129; -} -else -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; -lean_dec(x_17); -lean_dec_ref(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); -lean_dec_ref(x_11); -lean_dec(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_8); -lean_dec_ref(x_7); -lean_dec(x_6); -lean_dec_ref(x_5); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_189 = lean_ctor_get(x_184, 0); -lean_inc(x_189); -if (lean_is_exclusive(x_184)) { - lean_ctor_release(x_184, 0); - x_190 = x_184; -} else { - lean_dec_ref(x_184); - x_190 = lean_box(0); -} -if (lean_is_scalar(x_190)) { - x_191 = lean_alloc_ctor(1, 1, 0); -} else { - x_191 = x_190; -} -lean_ctor_set(x_191, 0, x_189); -return x_191; -} -} -} -} -else -{ -uint8_t x_192; -lean_dec(x_17); -lean_dec_ref(x_16); -lean_dec(x_15); -lean_dec_ref(x_14); -lean_dec_ref(x_11); -lean_dec(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_8); -lean_dec_ref(x_7); -lean_dec(x_6); -lean_dec_ref(x_5); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -lean_dec(x_1); -x_192 = !lean_is_exclusive(x_130); -if (x_192 == 0) -{ -return x_130; -} -else -{ -lean_object* x_193; lean_object* x_194; -x_193 = lean_ctor_get(x_130, 0); -lean_inc(x_193); -lean_dec(x_130); -x_194 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_194, 0, x_193); -return x_194; -} -} -block_48: -{ -uint8_t x_28; uint8_t x_29; lean_object* x_30; -x_28 = 0; -x_29 = 1; -x_30 = l_Lean_Meta_mkLambdaFVars(x_19, x_20, x_28, x_2, x_28, x_2, x_29, x_23, x_24, x_25, x_26); -lean_dec_ref(x_19); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -lean_dec_ref(x_30); -x_32 = lean_array_push(x_3, x_4); -x_33 = l_Lean_Meta_mkLambdaFVars(x_32, x_31, x_28, x_2, x_28, x_2, x_29, x_23, x_24, x_25, x_26); -lean_dec(x_26); -lean_dec_ref(x_25); -lean_dec(x_24); -lean_dec_ref(x_23); -lean_dec_ref(x_32); -if (lean_obj_tag(x_33) == 0) -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_33, 0); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_21); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_22); -lean_ctor_set(x_33, 0, x_37); -return x_33; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_33, 0); -lean_inc(x_38); -lean_dec(x_33); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_21); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_22); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -return x_41; -} -} -else -{ -uint8_t x_42; -lean_dec_ref(x_22); -lean_dec_ref(x_21); -x_42 = !lean_is_exclusive(x_33); -if (x_42 == 0) -{ -return x_33; -} -else -{ -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_33, 0); -lean_inc(x_43); -lean_dec(x_33); -x_44 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_44, 0, x_43); -return x_44; -} -} -} -else -{ -uint8_t x_45; -lean_dec(x_26); -lean_dec_ref(x_25); -lean_dec(x_24); -lean_dec_ref(x_23); -lean_dec_ref(x_22); -lean_dec_ref(x_21); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_45 = !lean_is_exclusive(x_30); -if (x_45 == 0) -{ -return x_30; -} -else -{ -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_30, 0); -lean_inc(x_46); -lean_dec(x_30); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_46); -return x_47; -} -} -} -block_129: -{ -lean_object* x_56; lean_object* x_57; -x_56 = l_Subarray_toArray___redArg(x_5); -lean_inc(x_54); -lean_inc_ref(x_53); -lean_inc(x_52); -lean_inc_ref(x_51); -x_57 = l_Lean_Meta_instantiateLambda(x_11, x_56, x_51, x_52, x_53, x_54); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec_ref(x_57); -lean_inc(x_58); -lean_inc(x_10); -lean_inc_ref(x_4); -x_59 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__1___boxed), 13, 5); -lean_closure_set(x_59, 0, x_4); -lean_closure_set(x_59, 1, x_10); -lean_closure_set(x_59, 2, x_6); -lean_closure_set(x_59, 3, x_7); -lean_closure_set(x_59, 4, x_58); -x_60 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_rwFun___boxed), 7, 1); -lean_closure_set(x_60, 0, x_8); -x_61 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_inProdLambdaLastArg___boxed), 7, 1); -lean_closure_set(x_61, 0, x_60); -lean_inc(x_54); -lean_inc_ref(x_53); -lean_inc(x_52); -lean_inc_ref(x_51); -x_62 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_withRewrittenMotive(x_9, x_61, x_59, x_49, x_50, x_51, x_52, x_53, x_54); -if (lean_obj_tag(x_62) == 0) -{ -lean_object* x_63; uint8_t x_64; -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -lean_dec_ref(x_62); -x_64 = !lean_is_exclusive(x_63); -if (x_64 == 0) -{ -lean_object* x_65; uint8_t x_66; -x_65 = lean_ctor_get(x_63, 0); -x_66 = !lean_is_exclusive(x_65); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_67 = lean_ctor_get(x_63, 1); -x_68 = lean_ctor_get(x_65, 0); -x_69 = lean_ctor_get(x_65, 1); -x_70 = l_Lean_Expr_containsFVar(x_68, x_10); -if (x_70 == 0) -{ -lean_free_object(x_65); -lean_free_object(x_63); -lean_dec(x_58); -lean_dec(x_10); -x_19 = x_56; -x_20 = x_68; -x_21 = x_69; -x_22 = x_67; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -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_dec(x_69); -lean_dec(x_67); -x_71 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__1; -x_72 = l_Lean_mkFVar(x_10); -x_73 = l_Lean_MessageData_ofExpr(x_72); -lean_ctor_set_tag(x_65, 7); -lean_ctor_set(x_65, 1, x_73); -lean_ctor_set(x_65, 0, x_71); -x_74 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__3; -lean_ctor_set_tag(x_63, 7); -lean_ctor_set(x_63, 1, x_74); -x_75 = l_Lean_indentExpr(x_58); -x_76 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_76, 0, x_63); -lean_ctor_set(x_76, 1, x_75); -x_77 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__0___redArg(x_76, x_51, x_52, x_53, x_54); -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); -lean_dec_ref(x_77); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -lean_dec(x_78); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -x_19 = x_56; -x_20 = x_68; -x_21 = x_81; -x_22 = x_80; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -else -{ -uint8_t x_82; -lean_dec(x_68); -lean_dec_ref(x_56); -lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); -lean_dec_ref(x_51); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_82 = !lean_is_exclusive(x_77); -if (x_82 == 0) -{ -return x_77; -} -else -{ -lean_object* x_83; lean_object* x_84; -x_83 = lean_ctor_get(x_77, 0); -lean_inc(x_83); -lean_dec(x_77); -x_84 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_84, 0, x_83); -return x_84; -} -} -} -} -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; -x_85 = lean_ctor_get(x_63, 1); -x_86 = lean_ctor_get(x_65, 0); -x_87 = lean_ctor_get(x_65, 1); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_65); -x_88 = l_Lean_Expr_containsFVar(x_86, x_10); -if (x_88 == 0) -{ -lean_free_object(x_63); -lean_dec(x_58); -lean_dec(x_10); -x_19 = x_56; -x_20 = x_86; -x_21 = x_87; -x_22 = x_85; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -else -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_87); -lean_dec(x_85); -x_89 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__1; -x_90 = l_Lean_mkFVar(x_10); -x_91 = l_Lean_MessageData_ofExpr(x_90); -x_92 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_92, 0, x_89); -lean_ctor_set(x_92, 1, x_91); -x_93 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__3; -lean_ctor_set_tag(x_63, 7); -lean_ctor_set(x_63, 1, x_93); -lean_ctor_set(x_63, 0, x_92); -x_94 = l_Lean_indentExpr(x_58); -x_95 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_95, 0, x_63); -lean_ctor_set(x_95, 1, x_94); -x_96 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__0___redArg(x_95, x_51, x_52, x_53, x_54); -if (lean_obj_tag(x_96) == 0) -{ -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -lean_dec_ref(x_96); -x_98 = lean_ctor_get(x_97, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_97, 1); -lean_inc(x_99); -lean_dec(x_97); -x_100 = lean_ctor_get(x_98, 1); -lean_inc(x_100); -lean_dec(x_98); -x_19 = x_56; -x_20 = x_86; -x_21 = x_100; -x_22 = x_99; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -else -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_86); -lean_dec_ref(x_56); -lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); -lean_dec_ref(x_51); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_101 = lean_ctor_get(x_96, 0); -lean_inc(x_101); -if (lean_is_exclusive(x_96)) { - lean_ctor_release(x_96, 0); - x_102 = x_96; -} else { - lean_dec_ref(x_96); - x_102 = lean_box(0); -} -if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 1, 0); -} else { - x_103 = x_102; -} -lean_ctor_set(x_103, 0, x_101); -return x_103; -} -} -} -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; -x_104 = lean_ctor_get(x_63, 0); -x_105 = lean_ctor_get(x_63, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_63); -x_106 = lean_ctor_get(x_104, 0); -lean_inc(x_106); -x_107 = lean_ctor_get(x_104, 1); -lean_inc(x_107); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_108 = x_104; -} else { - lean_dec_ref(x_104); - x_108 = lean_box(0); -} -x_109 = l_Lean_Expr_containsFVar(x_106, x_10); -if (x_109 == 0) -{ -lean_dec(x_108); -lean_dec(x_58); -lean_dec(x_10); -x_19 = x_56; -x_20 = x_106; -x_21 = x_107; -x_22 = x_105; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -else -{ -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -lean_dec(x_107); -lean_dec(x_105); -x_110 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__1; -x_111 = l_Lean_mkFVar(x_10); -x_112 = l_Lean_MessageData_ofExpr(x_111); -if (lean_is_scalar(x_108)) { - x_113 = lean_alloc_ctor(7, 2, 0); -} else { - x_113 = x_108; - lean_ctor_set_tag(x_113, 7); -} -lean_ctor_set(x_113, 0, x_110); -lean_ctor_set(x_113, 1, x_112); -x_114 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize___lam__5___closed__3; -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_indentExpr(x_58); -x_117 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_117, 0, x_115); -lean_ctor_set(x_117, 1, x_116); -x_118 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__0___redArg(x_117, x_51, x_52, x_53, x_54); -if (lean_obj_tag(x_118) == 0) -{ -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -lean_dec_ref(x_118); -x_120 = lean_ctor_get(x_119, 0); -lean_inc(x_120); -x_121 = lean_ctor_get(x_119, 1); -lean_inc(x_121); -lean_dec(x_119); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -lean_dec(x_120); -x_19 = x_56; -x_20 = x_106; -x_21 = x_122; -x_22 = x_121; -x_23 = x_51; -x_24 = x_52; -x_25 = x_53; -x_26 = x_54; -x_27 = lean_box(0); -goto block_48; -} -else -{ -lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_dec(x_106); -lean_dec_ref(x_56); -lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); -lean_dec_ref(x_51); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_123 = lean_ctor_get(x_118, 0); -lean_inc(x_123); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - x_124 = x_118; -} else { - lean_dec_ref(x_118); - x_124 = lean_box(0); -} -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(1, 1, 0); -} else { - x_125 = x_124; -} -lean_ctor_set(x_125, 0, x_123); -return x_125; -} -} -} -} -else -{ -lean_dec(x_58); -lean_dec_ref(x_56); -lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); -lean_dec_ref(x_51); -lean_dec(x_10); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -return x_62; -} -} -else -{ -uint8_t x_126; -lean_dec_ref(x_56); -lean_dec(x_54); -lean_dec_ref(x_53); -lean_dec(x_52); -lean_dec_ref(x_51); -lean_dec_ref(x_50); -lean_dec_ref(x_49); -lean_dec(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_8); -lean_dec_ref(x_7); -lean_dec(x_6); -lean_dec_ref(x_4); -lean_dec_ref(x_3); -x_126 = !lean_is_exclusive(x_57); -if (x_126 == 0) -{ -return x_57; -} -else -{ -lean_object* x_127; lean_object* x_128; -x_127 = lean_ctor_get(x_57, 0); -lean_inc(x_127); -lean_dec(x_57); -x_128 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_128, 0, x_127); -return x_128; -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -_start: -{ -uint8_t x_19; lean_object* x_20; -x_19 = lean_unbox(x_2); -x_20 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2(x_1, x_19, 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); -return x_20; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(".brecOn argument has too few parameters, expected at least ", 59, 59); -return x_1; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(": ", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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) { -_start: -{ -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_37; lean_object* x_38; lean_object* x_39; lean_object* x_50; uint8_t x_51; -x_50 = lean_array_get_size(x_9); -x_51 = lean_nat_dec_le(x_1, x_50); -if (x_51 == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_dec_ref(x_12); -lean_dec_ref(x_11); -x_52 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1; -lean_inc(x_1); -x_53 = l_Nat_reprFast(x_1); -x_54 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_54, 0, x_53); -x_55 = l_Lean_MessageData_ofFormat(x_54); -x_56 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_56, 0, x_52); -lean_ctor_set(x_56, 1, x_55); -x_57 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -lean_inc_ref(x_9); -x_59 = lean_array_to_list(x_9); -x_60 = lean_box(0); -x_61 = l_List_mapTR_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__4(x_59, x_60); -x_62 = l_Lean_MessageData_ofList(x_61); -x_63 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_63, 0, x_58); -lean_ctor_set(x_63, 1, x_62); -x_64 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__0___redArg(x_63, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_64) == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -lean_dec_ref(x_64); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_37 = x_68; -x_38 = x_67; -x_39 = lean_box(0); -goto block_49; +{ +lean_object* x_3; +x_3 = l_Array_finIdxOf_x3f___at___00Array_idxOf_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__11_spec__18(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = lean_box(0); +return x_4; } else { -uint8_t x_69; -lean_dec(x_16); -lean_dec_ref(x_15); -lean_dec(x_14); -lean_dec_ref(x_13); -lean_dec_ref(x_10); -lean_dec_ref(x_9); -lean_dec_ref(x_7); -lean_dec_ref(x_6); -lean_dec(x_4); -lean_dec_ref(x_3); -lean_dec_ref(x_2); -lean_dec(x_1); -x_69 = !lean_is_exclusive(x_64); -if (x_69 == 0) +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) { -return x_64; +return x_3; } else { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_64, 0); -lean_inc(x_70); -lean_dec(x_64); -x_71 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_71, 0, x_70); -return x_71; +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_6); +return x_7; +} +} } } +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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, uint8_t x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = l_Lean_Expr_getAppFn(x_9); +x_11 = l_Array_idxOf_x3f___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__11(x_1, x_10); +lean_dec_ref(x_10); +if (lean_obj_tag(x_11) == 1) +{ +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_11, 0); +lean_inc(x_12); +if (lean_is_exclusive(x_11)) { + lean_ctor_release(x_11, 0); + x_13 = x_11; +} else { + lean_dec_ref(x_11); + x_13 = lean_box(0); +} +x_14 = l_Lean_Expr_getAppNumArgs(x_9); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_array_get_borrowed(x_15, x_2, x_12); +x_17 = lean_nat_dec_eq(x_14, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec_ref(x_9); +lean_dec_ref(x_5); +lean_dec_ref(x_3); +x_18 = lean_box(0); +return x_18; } else { -x_37 = x_11; -x_38 = x_12; -x_39 = lean_box(0); -goto block_49; +lean_object* x_19; lean_object* x_20; +x_19 = lean_array_get_borrowed(x_3, x_4, x_12); +if (x_8 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_32 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0___lam__1___closed__0; +lean_inc(x_14); +x_33 = lean_mk_array(x_14, x_32); +x_34 = lean_unsigned_to_nat(1u); +x_35 = lean_nat_sub(x_14, x_34); +lean_dec(x_14); +x_36 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_33, x_35); +x_20 = x_36; +goto block_31; } -block_36: +else { -lean_object* x_25; -lean_inc(x_16); -lean_inc_ref(x_15); +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 = l___private_Lean_Meta_Transform_0__Lean_Core_transform_visit___at___00Lean_Core_transform___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_elimTypeAnnotations_spec__0_spec__0___lam__1___closed__0; lean_inc(x_14); -lean_inc_ref(x_13); -x_25 = l_Lean_Meta_instantiateLambda(x_3, x_23, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_25) == 0) +x_38 = lean_mk_array(x_14, x_37); +x_39 = lean_unsigned_to_nat(1u); +x_40 = lean_nat_sub(x_14, x_39); +lean_dec(x_14); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_38, x_40); +x_42 = lean_array_pop(x_41); +x_20 = x_42; +goto block_31; +} +block_31: { -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_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_21, 0); +x_23 = lean_ctor_get(x_21, 1); +x_24 = lean_array_get_borrowed(x_5, x_6, x_12); +lean_dec(x_12); +lean_inc(x_24); +x_25 = l_Lean_Elab_FixedParamPerm_buildArgs___redArg(x_24, x_7, x_20); +x_26 = lean_box(0); +lean_inc(x_23); +x_27 = l_List_mapTR_loop___at___00Lean_mkConstWithLevelParams___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveUnaryInduction_doRealize_spec__2_spec__4(x_23, x_26); +lean_inc(x_22); +x_28 = l_Lean_Expr_const___override(x_22, x_27); +x_29 = l_Lean_mkAppN(x_28, x_25); lean_dec_ref(x_25); -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_24, 1); -lean_inc(x_28); -lean_dec_ref(x_24); -x_29 = l_Array_toSubarray___redArg(x_9, x_27, x_28); -x_30 = lean_box(x_5); -x_31 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___boxed), 18, 9); -lean_closure_set(x_31, 0, x_4); -lean_closure_set(x_31, 1, x_30); -lean_closure_set(x_31, 2, x_23); -lean_closure_set(x_31, 3, x_21); -lean_closure_set(x_31, 4, x_29); -lean_closure_set(x_31, 5, x_19); -lean_closure_set(x_31, 6, x_6); -lean_closure_set(x_31, 7, x_7); -lean_closure_set(x_31, 8, x_10); -x_32 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_lambdaTelescope1___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__9___redArg(x_26, x_31, x_20, x_18, x_13, x_14, x_15, x_16); -return x_32; +if (lean_is_scalar(x_13)) { + x_30 = lean_alloc_ctor(1, 1, 0); +} else { + x_30 = x_13; +} +lean_ctor_set(x_30, 0, x_29); +return x_30; +} +} } else { -uint8_t x_33; -lean_dec_ref(x_24); -lean_dec_ref(x_23); -lean_dec_ref(x_21); -lean_dec_ref(x_20); -lean_dec(x_19); -lean_dec_ref(x_18); -lean_dec(x_16); -lean_dec_ref(x_15); -lean_dec(x_14); -lean_dec_ref(x_13); -lean_dec_ref(x_10); +lean_object* x_43; +lean_dec(x_11); lean_dec_ref(x_9); +lean_dec_ref(x_5); +lean_dec_ref(x_3); +x_43 = lean_box(0); +return x_43; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_8); +x_11 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__0(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_10, x_9); lean_dec_ref(x_7); lean_dec_ref(x_6); -lean_dec(x_4); -x_33 = !lean_is_exclusive(x_25); -if (x_33 == 0) -{ -return x_25; +lean_dec_ref(x_4); +lean_dec_ref(x_2); +lean_dec_ref(x_1); +return x_11; } -else -{ -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_25, 0); -lean_inc(x_34); -lean_dec(x_25); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; } +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = l_Lean_Expr_fvarId_x21(x_1); +x_15 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody___lam__13___closed__2; +lean_inc(x_2); +x_16 = lean_array_push(x_15, x_2); +lean_inc(x_14); +x_17 = lean_array_push(x_16, x_14); +x_18 = lean_mk_empty_array_with_capacity(x_3); +x_19 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody(x_17, x_18, x_6, x_2, x_14, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12); +return x_19; } } -block_49: +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_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_40 = lean_unsigned_to_nat(0u); -lean_inc(x_1); -lean_inc_ref(x_9); -x_41 = l_Array_toSubarray___redArg(x_9, x_40, x_1); -x_42 = l_Subarray_toArray___redArg(x_41); -x_43 = lean_array_get_borrowed(x_2, x_9, x_1); -x_44 = lean_array_get_size(x_9); -x_45 = lean_nat_add(x_1, x_8); -lean_dec(x_1); -x_46 = lean_nat_dec_le(x_45, x_40); -if (x_46 == 0) +lean_object* x_14; +x_14 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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_ref(x_1); +return x_14; +} +} +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0() { +_start: { -lean_object* x_47; -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_44); -lean_inc(x_43); -x_18 = x_38; -x_19 = x_40; -x_20 = x_37; -x_21 = x_43; -x_22 = lean_box(0); -x_23 = x_42; -x_24 = x_47; -goto block_36; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("replacing ", 10, 10); +return x_1; } -else +} +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1() { +_start: { -lean_object* x_48; -lean_dec(x_45); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_40); -lean_ctor_set(x_48, 1, x_44); -lean_inc(x_43); -x_18 = x_38; -x_19 = x_40; -x_20 = x_37; -x_21 = x_43; -x_22 = lean_box(0); -x_23 = x_42; -x_24 = x_48; -goto block_36; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" with ", 6, 6); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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]; +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3() { _start: { -uint8_t x_18; lean_object* x_19; -x_18 = lean_unbox(x_5); -x_19 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3(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); -lean_dec(x_8); -return x_19; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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_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_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_130; @@ -98051,14 +96899,14 @@ lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; x_141 = lean_ctor_get(x_132, 1); x_142 = lean_ctor_get(x_132, 0); lean_dec(x_142); -x_143 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; +x_143 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1; lean_inc(x_10); x_144 = l_Lean_Expr_fvar___override(x_10); x_145 = l_Lean_MessageData_ofExpr(x_144); lean_ctor_set_tag(x_132, 7); lean_ctor_set(x_132, 1, x_145); lean_ctor_set(x_132, 0, x_143); -x_146 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; +x_146 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3; lean_ctor_set_tag(x_131, 7); lean_ctor_set(x_131, 1, x_146); lean_inc_ref(x_4); @@ -98129,14 +96977,14 @@ lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; x_157 = lean_ctor_get(x_132, 1); lean_inc(x_157); lean_dec(x_132); -x_158 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; +x_158 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1; lean_inc(x_10); x_159 = l_Lean_Expr_fvar___override(x_10); x_160 = l_Lean_MessageData_ofExpr(x_159); x_161 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_161, 0, x_158); lean_ctor_set(x_161, 1, x_160); -x_162 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; +x_162 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3; lean_ctor_set_tag(x_131, 7); lean_ctor_set(x_131, 1, x_162); lean_ctor_set(x_131, 0, x_161); @@ -98220,7 +97068,7 @@ if (lean_is_exclusive(x_132)) { lean_dec_ref(x_132); x_175 = lean_box(0); } -x_176 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1; +x_176 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1; lean_inc(x_10); x_177 = l_Lean_Expr_fvar___override(x_10); x_178 = l_Lean_MessageData_ofExpr(x_177); @@ -98232,7 +97080,7 @@ if (lean_is_scalar(x_175)) { } lean_ctor_set(x_179, 0, x_176); lean_ctor_set(x_179, 1, x_178); -x_180 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3; +x_180 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3; x_181 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_181, 0, x_179); lean_ctor_set(x_181, 1, x_180); @@ -98850,7 +97698,7 @@ return x_128; } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -98873,11 +97721,45 @@ lean_object* x_18 = _args[17]; { uint8_t x_19; lean_object* x_20; x_19 = lean_unbox(x_2); -x_20 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2(x_1, x_19, 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_20 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2(x_1, x_19, 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); return x_20; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0(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) { +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(".brecOn argument has too few parameters, expected at least ", 59, 59); +return x_1; +} +} +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(": ", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__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) { _start: { 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_37; lean_object* x_38; lean_object* x_39; lean_object* x_50; uint8_t x_51; @@ -98888,7 +97770,7 @@ if (x_51 == 0) lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec_ref(x_12); lean_dec_ref(x_11); -x_52 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1; +x_52 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1; lean_inc(x_1); x_53 = l_Nat_reprFast(x_1); x_54 = lean_alloc_ctor(3, 1, 0); @@ -98897,7 +97779,7 @@ x_55 = l_Lean_MessageData_ofFormat(x_54); x_56 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_56, 0, x_52); lean_ctor_set(x_56, 1, x_55); -x_57 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; +x_57 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; x_58 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_58, 0, x_56); lean_ctor_set(x_58, 1, x_57); @@ -98975,7 +97857,7 @@ lean_inc(x_16); lean_inc_ref(x_15); lean_inc(x_14); lean_inc_ref(x_13); -x_25 = l_Lean_Meta_instantiateLambda(x_3, x_22, x_13, x_14, x_15, x_16); +x_25 = l_Lean_Meta_instantiateLambda(x_3, x_20, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_25) == 0) { lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; @@ -98989,17 +97871,17 @@ lean_inc(x_28); lean_dec_ref(x_24); x_29 = l_Array_toSubarray___redArg(x_9, x_27, x_28); x_30 = lean_box(x_5); -x_31 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___boxed), 18, 9); +x_31 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___boxed), 18, 9); lean_closure_set(x_31, 0, x_4); lean_closure_set(x_31, 1, x_30); -lean_closure_set(x_31, 2, x_22); -lean_closure_set(x_31, 3, x_18); +lean_closure_set(x_31, 2, x_20); +lean_closure_set(x_31, 3, x_22); lean_closure_set(x_31, 4, x_29); lean_closure_set(x_31, 5, x_19); lean_closure_set(x_31, 6, x_6); lean_closure_set(x_31, 7, x_7); lean_closure_set(x_31, 8, x_10); -x_32 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_lambdaTelescope1___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__9___redArg(x_26, x_31, x_23, x_20, x_13, x_14, x_15, x_16); +x_32 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_lambdaTelescope1___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_buildInductionBody_spec__9___redArg(x_26, x_31, x_21, x_23, x_13, x_14, x_15, x_16); return x_32; } else @@ -99008,9 +97890,9 @@ uint8_t x_33; lean_dec_ref(x_24); lean_dec_ref(x_23); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_20); lean_dec(x_19); -lean_dec_ref(x_18); lean_dec(x_16); lean_dec_ref(x_15); lean_dec(x_14); @@ -99057,12 +97939,12 @@ x_47 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_44); lean_inc(x_43); -x_18 = x_43; +x_18 = lean_box(0); x_19 = x_40; -x_20 = x_38; -x_21 = lean_box(0); -x_22 = x_42; -x_23 = x_37; +x_20 = x_42; +x_21 = x_37; +x_22 = x_43; +x_23 = x_38; x_24 = x_47; goto block_36; } @@ -99074,19 +97956,19 @@ x_48 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_48, 0, x_40); lean_ctor_set(x_48, 1, x_44); lean_inc(x_43); -x_18 = x_43; +x_18 = lean_box(0); x_19 = x_40; -x_20 = x_38; -x_21 = lean_box(0); -x_22 = x_42; -x_23 = x_37; +x_20 = x_42; +x_21 = x_37; +x_22 = x_43; +x_23 = x_38; x_24 = x_48; goto block_36; } } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -99108,7 +97990,7 @@ lean_object* x_17 = _args[16]; { uint8_t x_18; lean_object* x_19; x_18 = lean_unbox(x_5); -x_19 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0(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 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3(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); lean_dec(x_8); return x_19; } @@ -99281,7 +98163,7 @@ x_65 = lean_box(x_56); lean_inc_ref(x_10); lean_inc(x_11); lean_inc_ref(x_1); -x_66 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed), 17, 8); +x_66 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed), 17, 8); lean_closure_set(x_66, 0, x_64); lean_closure_set(x_66, 1, x_1); lean_closure_set(x_66, 2, x_63); @@ -99397,7 +98279,7 @@ x_87 = lean_box(x_56); lean_inc_ref(x_10); lean_inc(x_11); lean_inc_ref(x_1); -x_88 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed), 17, 8); +x_88 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed), 17, 8); lean_closure_set(x_88, 0, x_86); lean_closure_set(x_88, 1, x_1); lean_closure_set(x_88, 2, x_85); @@ -99570,7 +98452,7 @@ x_118 = lean_box(x_112); lean_inc_ref(x_10); lean_inc(x_11); lean_inc_ref(x_1); -x_119 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed), 17, 8); +x_119 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed), 17, 8); lean_closure_set(x_119, 0, x_117); lean_closure_set(x_119, 1, x_1); lean_closure_set(x_119, 2, x_116); @@ -99806,7 +98688,7 @@ x_157 = lean_box(x_150); lean_inc_ref(x_10); lean_inc(x_11); lean_inc_ref(x_1); -x_158 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed), 17, 8); +x_158 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed), 17, 8); lean_closure_set(x_158, 0, x_156); lean_closure_set(x_158, 1, x_1); lean_closure_set(x_158, 2, x_155); @@ -100065,7 +98947,7 @@ x_201 = lean_box(x_193); lean_inc_ref(x_10); lean_inc(x_11); lean_inc_ref(x_1); -x_202 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___boxed), 17, 8); +x_202 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___boxed), 17, 8); lean_closure_set(x_202, 0, x_200); lean_closure_set(x_202, 1, x_1); lean_closure_set(x_202, 2, x_199); @@ -101550,21 +100432,21 @@ goto block_41; uint8_t x_20; uint8_t x_21; lean_object* x_22; x_20 = 0; x_21 = 1; -x_22 = l_Lean_Meta_mkForallFVars(x_18, x_19, x_20, x_1, x_1, x_21, x_12, x_13, x_14, x_15); -lean_dec_ref(x_18); +x_22 = l_Lean_Meta_mkForallFVars(x_17, x_19, x_20, x_1, x_1, x_21, x_12, x_13, x_14, x_15); +lean_dec_ref(x_17); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); lean_dec_ref(x_22); -x_24 = l_Lean_Meta_mkLambdaFVars(x_17, x_23, x_20, x_1, x_20, x_1, x_21, x_12, x_13, x_14, x_15); -lean_dec_ref(x_17); +x_24 = l_Lean_Meta_mkLambdaFVars(x_18, x_23, x_20, x_1, x_20, x_1, x_21, x_12, x_13, x_14, x_15); +lean_dec_ref(x_18); return x_24; } else { -lean_dec_ref(x_17); +lean_dec_ref(x_18); return x_22; } } @@ -101584,8 +100466,8 @@ if (x_4 == 0) lean_dec_ref(x_26); lean_dec_ref(x_6); lean_dec_ref(x_5); -x_17 = x_28; -x_18 = x_29; +x_17 = x_29; +x_18 = x_28; x_19 = x_30; goto block_25; } @@ -101609,8 +100491,8 @@ x_38 = l_Lean_Expr_const___override(x_32, x_37); x_39 = l_Lean_mkAppN(x_38, x_35); lean_dec_ref(x_35); x_40 = l_Lean_Expr_app___override(x_30, x_39); -x_17 = x_28; -x_18 = x_29; +x_17 = x_29; +x_18 = x_28; x_19 = x_40; goto block_25; } @@ -103141,7 +102023,7 @@ x_59 = l_Lean_MessageData_ofName(x_13); lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_59); lean_ctor_set(x_35, 0, x_58); -x_60 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; +x_60 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; lean_ctor_set_tag(x_24, 7); lean_ctor_set(x_24, 1, x_60); lean_ctor_set(x_24, 0, x_35); @@ -103229,7 +102111,7 @@ x_74 = l_Lean_MessageData_ofName(x_13); lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_74); lean_ctor_set(x_35, 0, x_73); -x_75 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; +x_75 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; lean_ctor_set_tag(x_24, 7); lean_ctor_set(x_24, 1, x_75); lean_ctor_set(x_24, 0, x_35); @@ -103490,7 +102372,7 @@ x_111 = l_Lean_MessageData_ofName(x_13); x_112 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_112, 0, x_110); lean_ctor_set(x_112, 1, x_111); -x_113 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; +x_113 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; lean_ctor_set_tag(x_24, 7); lean_ctor_set(x_24, 1, x_113); lean_ctor_set(x_24, 0, x_112); @@ -103794,7 +102676,7 @@ if (lean_is_scalar(x_140)) { } lean_ctor_set(x_163, 0, x_161); lean_ctor_set(x_163, 1, x_162); -x_164 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3; +x_164 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3; x_165 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_165, 0, x_163); lean_ctor_set(x_165, 1, x_164); @@ -107586,8 +106468,8 @@ lean_dec_ref(x_71); lean_dec(x_70); lean_dec_ref(x_69); lean_dec(x_13); -x_32 = x_91; -x_33 = x_94; +x_32 = x_94; +x_33 = x_91; x_34 = lean_box(0); goto block_38; } @@ -107608,8 +106490,8 @@ lean_dec_ref(x_69); if (lean_obj_tag(x_100) == 0) { lean_dec_ref(x_100); -x_32 = x_91; -x_33 = x_94; +x_32 = x_94; +x_33 = x_91; x_34 = lean_box(0); goto block_38; } @@ -107663,8 +106545,8 @@ lean_dec_ref(x_71); lean_dec(x_70); lean_dec_ref(x_69); lean_dec(x_13); -x_32 = x_104; -x_33 = x_107; +x_32 = x_107; +x_33 = x_104; x_34 = lean_box(0); goto block_38; } @@ -107685,8 +106567,8 @@ lean_dec_ref(x_69); if (lean_obj_tag(x_114) == 0) { lean_dec_ref(x_114); -x_32 = x_104; -x_33 = x_107; +x_32 = x_107; +x_33 = x_104; x_34 = lean_box(0); goto block_38; } @@ -108375,10 +107257,10 @@ return x_229; { lean_object* x_35; lean_object* x_36; lean_object* x_37; x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_32); +lean_ctor_set(x_35, 0, x_33); lean_ctor_set(x_35, 1, x_14); x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_33); +lean_ctor_set(x_36, 0, x_32); lean_ctor_set(x_36, 1, x_35); x_37 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_37, 0, x_36); @@ -109842,17 +108724,17 @@ goto block_353; lean_object* x_52; lean_object* x_53; uint8_t x_54; x_52 = lean_array_get_size(x_46); lean_dec_ref(x_46); -x_53 = lean_array_get_size(x_43); +x_53 = lean_array_get_size(x_45); x_54 = lean_nat_dec_eq(x_52, x_53); if (x_54 == 0) { lean_object* x_55; lean_object* x_56; lean_dec_ref(x_45); -lean_dec(x_44); +lean_dec_ref(x_44); lean_dec_ref(x_43); -lean_dec(x_42); -lean_dec_ref(x_41); -lean_dec_ref(x_40); +lean_dec_ref(x_42); +lean_dec(x_41); +lean_dec(x_40); lean_dec_ref(x_39); lean_dec_ref(x_38); lean_dec_ref(x_37); @@ -109886,28 +108768,28 @@ x_63 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_FunInd_0__Lean_Ta lean_closure_set(x_63, 0, x_4); lean_closure_set(x_63, 1, x_5); lean_closure_set(x_63, 2, x_6); -lean_closure_set(x_63, 3, x_36); +lean_closure_set(x_63, 3, x_41); lean_closure_set(x_63, 4, x_60); lean_closure_set(x_63, 5, x_7); lean_closure_set(x_63, 6, x_1); lean_closure_set(x_63, 7, x_2); lean_closure_set(x_63, 8, x_59); -lean_closure_set(x_63, 9, x_44); +lean_closure_set(x_63, 9, x_40); lean_closure_set(x_63, 10, x_61); lean_closure_set(x_63, 11, x_33); -lean_closure_set(x_63, 12, x_34); -lean_closure_set(x_63, 13, x_43); -lean_closure_set(x_63, 14, x_37); -lean_closure_set(x_63, 15, x_41); -lean_closure_set(x_63, 16, x_45); +lean_closure_set(x_63, 12, x_39); +lean_closure_set(x_63, 13, x_45); +lean_closure_set(x_63, 14, x_44); +lean_closure_set(x_63, 15, x_43); +lean_closure_set(x_63, 16, x_42); lean_closure_set(x_63, 17, x_62); -lean_closure_set(x_63, 18, x_40); +lean_closure_set(x_63, 18, x_35); lean_closure_set(x_63, 19, x_38); lean_closure_set(x_63, 20, x_10); lean_closure_set(x_63, 21, x_11); -lean_closure_set(x_63, 22, x_35); -lean_closure_set(x_63, 23, x_39); -lean_closure_set(x_63, 24, x_42); +lean_closure_set(x_63, 22, x_37); +lean_closure_set(x_63, 23, x_34); +lean_closure_set(x_63, 24, x_36); x_64 = l_Lean_Meta_withErasedFVars___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__18___redArg(x_58, x_63, x_47, x_48, x_49, x_50); lean_dec_ref(x_58); return x_64; @@ -109926,27 +108808,27 @@ lean_object* x_79; lean_object* x_80; uint8_t x_81; x_79 = lean_ctor_get(x_26, 1); x_80 = lean_ctor_get(x_26, 0); lean_dec(x_80); -x_81 = !lean_is_exclusive(x_70); +x_81 = !lean_is_exclusive(x_71); if (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_70, 0); -x_83 = lean_ctor_get(x_70, 2); +x_82 = lean_ctor_get(x_71, 0); +x_83 = lean_ctor_get(x_71, 2); lean_dec(x_83); -x_84 = lean_ctor_get(x_70, 1); +x_84 = lean_ctor_get(x_71, 1); lean_dec(x_84); x_85 = l_Lean_Level_ofNat(x_2); lean_inc(x_79); lean_inc(x_85); lean_ctor_set(x_26, 0, x_85); x_86 = l_Lean_Expr_const___override(x_82, x_26); -x_87 = l_Lean_mkAppN(x_86, x_71); +x_87 = l_Lean_mkAppN(x_86, x_72); lean_inc(x_76); lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); -lean_inc(x_69); -x_88 = l_Lean_Meta_inferArgumentTypesN(x_69, x_87, x_73, x_74, x_75, x_76); +lean_inc(x_70); +x_88 = l_Lean_Meta_inferArgumentTypesN(x_70, x_87, x_73, x_74, x_75, x_76); if (lean_obj_tag(x_88) == 0) { lean_object* x_89; size_t x_90; lean_object* x_91; @@ -109965,11 +108847,11 @@ lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; x_92 = lean_ctor_get(x_91, 0); lean_inc(x_92); lean_dec_ref(x_91); -lean_inc_ref(x_72); -x_93 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_72); -lean_ctor_set(x_70, 2, x_71); -lean_ctor_set(x_70, 1, x_79); -lean_ctor_set(x_70, 0, x_93); +lean_inc_ref(x_69); +x_93 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_69); +lean_ctor_set(x_71, 2, x_72); +lean_ctor_set(x_71, 1, x_79); +lean_ctor_set(x_71, 0, x_93); x_94 = lean_mk_empty_array_with_capacity(x_1); lean_inc(x_76); lean_inc_ref(x_75); @@ -109977,10 +108859,10 @@ lean_inc(x_74); lean_inc_ref(x_73); lean_inc(x_1); lean_inc(x_2); -lean_inc_ref(x_70); +lean_inc_ref(x_71); lean_inc_ref(x_6); lean_inc_ref(x_4); -x_95 = l_Array_mapFinIdxM_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__5___redArg(x_4, x_5, x_6, x_70, x_32, x_2, x_7, x_1, x_2, x_94, x_73, x_74, x_75, x_76); +x_95 = l_Array_mapFinIdxM_map___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__5___redArg(x_4, x_5, x_6, x_71, x_32, x_2, x_7, x_1, x_2, x_94, x_73, x_74, x_75, x_76); if (lean_obj_tag(x_95) == 0) { lean_object* x_96; lean_object* x_97; lean_object* x_98; @@ -109988,13 +108870,13 @@ x_96 = lean_ctor_get(x_95, 0); lean_inc(x_96); lean_dec_ref(x_95); lean_inc(x_85); -x_97 = l_Lean_Elab_Structural_IndGroupInst_brecOn(x_70, x_85, x_2); +x_97 = l_Lean_Elab_Structural_IndGroupInst_brecOn(x_71, x_85, x_2); lean_inc(x_76); lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); lean_inc_ref(x_97); -x_98 = l_Lean_Meta_inferArgumentTypesN(x_69, x_97, x_73, x_74, x_75, x_76); +x_98 = l_Lean_Meta_inferArgumentTypesN(x_70, x_97, x_73, x_74, x_75, x_76); 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; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; @@ -110008,8 +108890,8 @@ lean_inc(x_102); lean_dec_ref(x_101); x_103 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__6___closed__2; x_104 = lean_alloc_closure((void*)(l_instDecidableEqNat___boxed), 2, 0); -x_105 = l_Lean_InductiveVal_numTypeFormers(x_72); -lean_dec_ref(x_72); +x_105 = l_Lean_InductiveVal_numTypeFormers(x_69); +lean_dec_ref(x_69); x_106 = l_Array_range(x_105); x_107 = l_Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6___redArg(x_103, x_8, x_96, x_106); x_108 = lean_unbox(x_102); @@ -110017,18 +108899,18 @@ lean_dec(x_102); if (x_108 == 0) { lean_inc(x_99); -x_34 = x_96; -x_35 = x_66; -x_36 = x_85; -x_37 = x_99; -x_38 = x_67; -x_39 = x_97; -x_40 = x_92; -x_41 = x_104; -x_42 = x_68; -x_43 = x_107; -x_44 = x_100; -x_45 = x_70; +x_34 = x_97; +x_35 = x_92; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_96; +x_40 = x_100; +x_41 = x_85; +x_42 = x_71; +x_43 = x_104; +x_44 = x_99; +x_45 = x_107; x_46 = x_99; x_47 = x_73; x_48 = x_74; @@ -110054,18 +108936,18 @@ if (lean_obj_tag(x_115) == 0) { lean_dec_ref(x_115); lean_inc(x_99); -x_34 = x_96; -x_35 = x_66; -x_36 = x_85; -x_37 = x_99; -x_38 = x_67; -x_39 = x_97; -x_40 = x_92; -x_41 = x_104; -x_42 = x_68; -x_43 = x_107; -x_44 = x_100; -x_45 = x_70; +x_34 = x_97; +x_35 = x_92; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_96; +x_40 = x_100; +x_41 = x_85; +x_42 = x_71; +x_43 = x_104; +x_44 = x_99; +x_45 = x_107; x_46 = x_99; x_47 = x_73; x_48 = x_74; @@ -110082,7 +108964,7 @@ lean_dec_ref(x_104); lean_dec(x_99); lean_dec_ref(x_97); lean_dec(x_96); -lean_dec_ref(x_70); +lean_dec_ref(x_71); lean_dec(x_92); lean_dec(x_85); lean_dec(x_76); @@ -110125,14 +109007,14 @@ else uint8_t x_119; lean_dec_ref(x_97); lean_dec(x_96); -lean_dec_ref(x_70); +lean_dec_ref(x_71); lean_dec(x_92); lean_dec(x_85); lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110167,15 +109049,15 @@ return x_121; else { uint8_t x_122; -lean_dec_ref(x_70); +lean_dec_ref(x_71); lean_dec(x_92); lean_dec(x_85); lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110211,15 +109093,15 @@ else { uint8_t x_125; lean_dec(x_85); -lean_free_object(x_70); +lean_free_object(x_71); lean_dec(x_79); lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110255,15 +109137,15 @@ else { uint8_t x_128; lean_dec(x_85); -lean_free_object(x_70); +lean_free_object(x_71); lean_dec(x_79); lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110298,21 +109180,21 @@ return x_130; else { lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_131 = lean_ctor_get(x_70, 0); +x_131 = lean_ctor_get(x_71, 0); lean_inc(x_131); -lean_dec(x_70); +lean_dec(x_71); x_132 = l_Lean_Level_ofNat(x_2); lean_inc(x_79); lean_inc(x_132); lean_ctor_set(x_26, 0, x_132); x_133 = l_Lean_Expr_const___override(x_131, x_26); -x_134 = l_Lean_mkAppN(x_133, x_71); +x_134 = l_Lean_mkAppN(x_133, x_72); lean_inc(x_76); lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); -lean_inc(x_69); -x_135 = l_Lean_Meta_inferArgumentTypesN(x_69, x_134, x_73, x_74, x_75, x_76); +lean_inc(x_70); +x_135 = l_Lean_Meta_inferArgumentTypesN(x_70, x_134, x_73, x_74, x_75, x_76); if (lean_obj_tag(x_135) == 0) { lean_object* x_136; size_t x_137; lean_object* x_138; @@ -110331,12 +109213,12 @@ lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; x_139 = lean_ctor_get(x_138, 0); lean_inc(x_139); lean_dec_ref(x_138); -lean_inc_ref(x_72); -x_140 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_72); +lean_inc_ref(x_69); +x_140 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_69); x_141 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_141, 0, x_140); lean_ctor_set(x_141, 1, x_79); -lean_ctor_set(x_141, 2, x_71); +lean_ctor_set(x_141, 2, x_72); x_142 = lean_mk_empty_array_with_capacity(x_1); lean_inc(x_76); lean_inc_ref(x_75); @@ -110361,7 +109243,7 @@ lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); lean_inc_ref(x_145); -x_146 = l_Lean_Meta_inferArgumentTypesN(x_69, x_145, x_73, x_74, x_75, x_76); +x_146 = l_Lean_Meta_inferArgumentTypesN(x_70, x_145, x_73, x_74, x_75, x_76); 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; uint8_t x_156; @@ -110375,8 +109257,8 @@ lean_inc(x_150); lean_dec_ref(x_149); x_151 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__6___closed__2; x_152 = lean_alloc_closure((void*)(l_instDecidableEqNat___boxed), 2, 0); -x_153 = l_Lean_InductiveVal_numTypeFormers(x_72); -lean_dec_ref(x_72); +x_153 = l_Lean_InductiveVal_numTypeFormers(x_69); +lean_dec_ref(x_69); x_154 = l_Array_range(x_153); x_155 = l_Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6___redArg(x_151, x_8, x_144, x_154); x_156 = lean_unbox(x_150); @@ -110384,18 +109266,18 @@ lean_dec(x_150); if (x_156 == 0) { lean_inc(x_147); -x_34 = x_144; -x_35 = x_66; -x_36 = x_132; -x_37 = x_147; -x_38 = x_67; -x_39 = x_145; -x_40 = x_139; -x_41 = x_152; -x_42 = x_68; -x_43 = x_155; -x_44 = x_148; -x_45 = x_141; +x_34 = x_145; +x_35 = x_139; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_144; +x_40 = x_148; +x_41 = x_132; +x_42 = x_141; +x_43 = x_152; +x_44 = x_147; +x_45 = x_155; x_46 = x_147; x_47 = x_73; x_48 = x_74; @@ -110421,18 +109303,18 @@ if (lean_obj_tag(x_163) == 0) { lean_dec_ref(x_163); lean_inc(x_147); -x_34 = x_144; -x_35 = x_66; -x_36 = x_132; -x_37 = x_147; -x_38 = x_67; -x_39 = x_145; -x_40 = x_139; -x_41 = x_152; -x_42 = x_68; -x_43 = x_155; -x_44 = x_148; -x_45 = x_141; +x_34 = x_145; +x_35 = x_139; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_144; +x_40 = x_148; +x_41 = x_132; +x_42 = x_141; +x_43 = x_152; +x_44 = x_147; +x_45 = x_155; x_46 = x_147; x_47 = x_73; x_48 = x_74; @@ -110500,7 +109382,7 @@ lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110543,8 +109425,8 @@ lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110587,8 +109469,8 @@ lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110631,8 +109513,8 @@ lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110672,15 +109554,15 @@ lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; x_179 = lean_ctor_get(x_26, 1); lean_inc(x_179); lean_dec(x_26); -x_180 = lean_ctor_get(x_70, 0); +x_180 = lean_ctor_get(x_71, 0); lean_inc(x_180); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - lean_ctor_release(x_70, 2); - x_181 = x_70; +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + lean_ctor_release(x_71, 2); + x_181 = x_71; } else { - lean_dec_ref(x_70); + lean_dec_ref(x_71); x_181 = lean_box(0); } x_182 = l_Lean_Level_ofNat(x_2); @@ -110690,13 +109572,13 @@ x_183 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_183, 0, x_182); lean_ctor_set(x_183, 1, x_179); x_184 = l_Lean_Expr_const___override(x_180, x_183); -x_185 = l_Lean_mkAppN(x_184, x_71); +x_185 = l_Lean_mkAppN(x_184, x_72); lean_inc(x_76); lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); -lean_inc(x_69); -x_186 = l_Lean_Meta_inferArgumentTypesN(x_69, x_185, x_73, x_74, x_75, x_76); +lean_inc(x_70); +x_186 = l_Lean_Meta_inferArgumentTypesN(x_70, x_185, x_73, x_74, x_75, x_76); if (lean_obj_tag(x_186) == 0) { lean_object* x_187; size_t x_188; lean_object* x_189; @@ -110715,8 +109597,8 @@ lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; x_190 = lean_ctor_get(x_189, 0); lean_inc(x_190); lean_dec_ref(x_189); -lean_inc_ref(x_72); -x_191 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_72); +lean_inc_ref(x_69); +x_191 = l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(x_69); if (lean_is_scalar(x_181)) { x_192 = lean_alloc_ctor(0, 3, 0); } else { @@ -110724,7 +109606,7 @@ if (lean_is_scalar(x_181)) { } lean_ctor_set(x_192, 0, x_191); lean_ctor_set(x_192, 1, x_179); -lean_ctor_set(x_192, 2, x_71); +lean_ctor_set(x_192, 2, x_72); x_193 = lean_mk_empty_array_with_capacity(x_1); lean_inc(x_76); lean_inc_ref(x_75); @@ -110749,7 +109631,7 @@ lean_inc_ref(x_75); lean_inc(x_74); lean_inc_ref(x_73); lean_inc_ref(x_196); -x_197 = l_Lean_Meta_inferArgumentTypesN(x_69, x_196, x_73, x_74, x_75, x_76); +x_197 = l_Lean_Meta_inferArgumentTypesN(x_70, x_196, x_73, x_74, x_75, x_76); if (lean_obj_tag(x_197) == 0) { lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; @@ -110763,8 +109645,8 @@ lean_inc(x_201); lean_dec_ref(x_200); x_202 = l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__6___closed__2; x_203 = lean_alloc_closure((void*)(l_instDecidableEqNat___boxed), 2, 0); -x_204 = l_Lean_InductiveVal_numTypeFormers(x_72); -lean_dec_ref(x_72); +x_204 = l_Lean_InductiveVal_numTypeFormers(x_69); +lean_dec_ref(x_69); x_205 = l_Array_range(x_204); x_206 = l_Lean_Elab_Structural_Positions_groupAndSort___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__6___redArg(x_202, x_8, x_195, x_205); x_207 = lean_unbox(x_201); @@ -110772,18 +109654,18 @@ lean_dec(x_201); if (x_207 == 0) { lean_inc(x_198); -x_34 = x_195; -x_35 = x_66; -x_36 = x_182; -x_37 = x_198; -x_38 = x_67; -x_39 = x_196; -x_40 = x_190; -x_41 = x_203; -x_42 = x_68; -x_43 = x_206; -x_44 = x_199; -x_45 = x_192; +x_34 = x_196; +x_35 = x_190; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_195; +x_40 = x_199; +x_41 = x_182; +x_42 = x_192; +x_43 = x_203; +x_44 = x_198; +x_45 = x_206; x_46 = x_198; x_47 = x_73; x_48 = x_74; @@ -110809,18 +109691,18 @@ if (lean_obj_tag(x_214) == 0) { lean_dec_ref(x_214); lean_inc(x_198); -x_34 = x_195; -x_35 = x_66; -x_36 = x_182; -x_37 = x_198; -x_38 = x_67; -x_39 = x_196; -x_40 = x_190; -x_41 = x_203; -x_42 = x_68; -x_43 = x_206; -x_44 = x_199; -x_45 = x_192; +x_34 = x_196; +x_35 = x_190; +x_36 = x_68; +x_37 = x_67; +x_38 = x_66; +x_39 = x_195; +x_40 = x_199; +x_41 = x_182; +x_42 = x_192; +x_43 = x_203; +x_44 = x_198; +x_45 = x_206; x_46 = x_198; x_47 = x_73; x_48 = x_74; @@ -110888,7 +109770,7 @@ lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110931,8 +109813,8 @@ lean_dec(x_76); lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); -lean_dec_ref(x_72); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -110976,8 +109858,8 @@ lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -111021,8 +109903,8 @@ lean_dec_ref(x_75); lean_dec(x_74); lean_dec_ref(x_73); lean_dec_ref(x_72); -lean_dec_ref(x_71); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -111061,8 +109943,8 @@ else lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_dec_ref(x_72); lean_dec_ref(x_71); -lean_dec_ref(x_70); -lean_dec(x_69); +lean_dec(x_70); +lean_dec_ref(x_69); lean_dec(x_68); lean_dec_ref(x_67); lean_dec_ref(x_66); @@ -111094,18 +109976,18 @@ return x_233; block_259: { lean_object* x_248; uint8_t x_249; -x_248 = lean_array_get_size(x_241); +x_248 = lean_array_get_size(x_242); x_249 = lean_nat_dec_lt(x_2, x_248); if (x_249 == 0) { -lean_dec_ref(x_241); -x_66 = x_235; +lean_dec_ref(x_242); +x_66 = x_237; x_67 = x_236; -x_68 = x_237; +x_68 = x_235; x_69 = x_238; -x_70 = x_239; -x_71 = x_240; -x_72 = x_242; +x_70 = x_240; +x_71 = x_239; +x_72 = x_241; x_73 = x_243; x_74 = x_244; x_75 = x_245; @@ -111117,14 +109999,14 @@ else { if (x_249 == 0) { -lean_dec_ref(x_241); -x_66 = x_235; +lean_dec_ref(x_242); +x_66 = x_237; x_67 = x_236; -x_68 = x_237; +x_68 = x_235; x_69 = x_238; -x_70 = x_239; -x_71 = x_240; -x_72 = x_242; +x_70 = x_240; +x_71 = x_239; +x_72 = x_241; x_73 = x_243; x_74 = x_244; x_75 = x_245; @@ -111136,17 +110018,17 @@ else { size_t x_250; uint8_t x_251; x_250 = lean_usize_of_nat(x_248); -x_251 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__19(x_241, x_3, x_250); -lean_dec_ref(x_241); +x_251 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__19(x_242, x_3, x_250); +lean_dec_ref(x_242); if (x_251 == 0) { -x_66 = x_235; +x_66 = x_237; x_67 = x_236; -x_68 = x_237; +x_68 = x_235; x_69 = x_238; -x_70 = x_239; -x_71 = x_240; -x_72 = x_242; +x_70 = x_240; +x_71 = x_239; +x_72 = x_241; x_73 = x_243; x_74 = x_244; x_75 = x_245; @@ -111157,13 +110039,13 @@ goto block_234; else { lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; uint8_t x_256; -lean_dec_ref(x_242); -lean_dec_ref(x_240); +lean_dec_ref(x_241); +lean_dec(x_240); lean_dec_ref(x_239); -lean_dec(x_238); -lean_dec(x_237); +lean_dec_ref(x_238); +lean_dec_ref(x_237); lean_dec_ref(x_236); -lean_dec_ref(x_235); +lean_dec(x_235); lean_dec_ref(x_33); lean_dec(x_26); lean_dec_ref(x_14); @@ -111210,23 +110092,23 @@ return x_258; lean_object* x_280; lean_object* x_281; lean_object* x_282; uint8_t x_283; x_280 = l_Array_toSubarray___redArg(x_266, x_278, x_279); x_281 = l_Subarray_toArray___redArg(x_280); -x_282 = lean_array_get_size(x_268); +x_282 = lean_array_get_size(x_270); x_283 = lean_nat_dec_lt(x_2, x_282); if (x_283 == 0) { -lean_inc(x_271); +lean_inc(x_268); x_235 = x_268; -x_236 = x_269; -x_237 = x_271; -x_238 = x_271; -x_239 = x_267; -x_240 = x_270; -x_241 = x_281; -x_242 = x_276; -x_243 = x_273; -x_244 = x_272; -x_245 = x_275; -x_246 = x_274; +x_236 = x_270; +x_237 = x_267; +x_238 = x_275; +x_239 = x_269; +x_240 = x_268; +x_241 = x_271; +x_242 = x_281; +x_243 = x_277; +x_244 = x_273; +x_245 = x_274; +x_246 = x_276; x_247 = lean_box(0); goto block_259; } @@ -111234,19 +110116,19 @@ else { if (x_283 == 0) { -lean_inc(x_271); +lean_inc(x_268); x_235 = x_268; -x_236 = x_269; -x_237 = x_271; -x_238 = x_271; -x_239 = x_267; -x_240 = x_270; -x_241 = x_281; -x_242 = x_276; -x_243 = x_273; -x_244 = x_272; -x_245 = x_275; -x_246 = x_274; +x_236 = x_270; +x_237 = x_267; +x_238 = x_275; +x_239 = x_269; +x_240 = x_268; +x_241 = x_271; +x_242 = x_281; +x_243 = x_277; +x_244 = x_273; +x_245 = x_274; +x_246 = x_276; x_247 = lean_box(0); goto block_259; } @@ -111254,22 +110136,22 @@ else { size_t x_284; uint8_t x_285; x_284 = lean_usize_of_nat(x_282); -x_285 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__19(x_268, x_3, x_284); +x_285 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__19(x_270, x_3, x_284); if (x_285 == 0) { -lean_inc(x_271); +lean_inc(x_268); x_235 = x_268; -x_236 = x_269; -x_237 = x_271; -x_238 = x_271; -x_239 = x_267; -x_240 = x_270; -x_241 = x_281; -x_242 = x_276; -x_243 = x_273; -x_244 = x_272; -x_245 = x_275; -x_246 = x_274; +x_236 = x_270; +x_237 = x_267; +x_238 = x_275; +x_239 = x_269; +x_240 = x_268; +x_241 = x_271; +x_242 = x_281; +x_243 = x_277; +x_244 = x_273; +x_245 = x_274; +x_246 = x_276; x_247 = lean_box(0); goto block_259; } @@ -111277,11 +110159,11 @@ else { lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; uint8_t x_290; lean_dec_ref(x_281); -lean_dec_ref(x_276); -lean_dec(x_271); +lean_dec_ref(x_275); +lean_dec_ref(x_271); lean_dec_ref(x_270); lean_dec_ref(x_269); -lean_dec_ref(x_268); +lean_dec(x_268); lean_dec_ref(x_267); lean_dec_ref(x_33); lean_dec(x_26); @@ -111300,11 +110182,11 @@ x_287 = l_Lean_indentExpr(x_24); x_288 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_288, 0, x_286); lean_ctor_set(x_288, 1, x_287); -x_289 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__8___redArg(x_288, x_273, x_272, x_275, x_274); -lean_dec(x_274); -lean_dec_ref(x_275); -lean_dec(x_272); -lean_dec_ref(x_273); +x_289 = l_Lean_throwError___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_foldAndCollect_spec__8___redArg(x_288, x_277, x_273, x_274, x_276); +lean_dec(x_276); +lean_dec_ref(x_274); +lean_dec(x_273); +lean_dec_ref(x_277); x_290 = !lean_is_exclusive(x_289); if (x_290 == 0) { @@ -111351,17 +110233,17 @@ x_314 = lean_array_get_size(x_266); x_315 = lean_nat_dec_le(x_311, x_2); if (x_315 == 0) { -x_267 = x_295; -x_268 = x_310; -x_269 = x_313; -x_270 = x_305; -x_271 = x_298; -x_272 = x_300; -x_273 = x_299; -x_274 = x_302; -x_275 = x_301; -x_276 = x_294; -x_277 = lean_box(0); +x_267 = x_313; +x_268 = x_298; +x_269 = x_295; +x_270 = x_310; +x_271 = x_305; +x_272 = lean_box(0); +x_273 = x_300; +x_274 = x_301; +x_275 = x_294; +x_276 = x_302; +x_277 = x_299; x_278 = x_311; x_279 = x_314; goto block_293; @@ -111370,17 +110252,17 @@ else { lean_dec(x_311); lean_inc(x_2); -x_267 = x_295; -x_268 = x_310; -x_269 = x_313; -x_270 = x_305; -x_271 = x_298; -x_272 = x_300; -x_273 = x_299; -x_274 = x_302; -x_275 = x_301; -x_276 = x_294; -x_277 = lean_box(0); +x_267 = x_313; +x_268 = x_298; +x_269 = x_295; +x_270 = x_310; +x_271 = x_305; +x_272 = lean_box(0); +x_273 = x_300; +x_274 = x_301; +x_275 = x_294; +x_276 = x_302; +x_277 = x_299; x_278 = x_2; x_279 = x_314; goto block_293; @@ -114375,7 +113257,7 @@ x_47 = lean_unsigned_to_nat(5u); lean_inc_ref(x_4); x_48 = l_Array_toSubarray___redArg(x_4, x_46, x_47); x_49 = lean_box(0); -x_50 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_refinedArguments_go_spec__0___redArg(x_1, x_49, x_48, x_49, x_40, x_42, x_43, x_45, x_44); +x_50 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_refinedArguments_go_spec__0___redArg(x_1, x_49, x_48, x_49, x_41, x_42, x_43, x_44, x_45); if (lean_obj_tag(x_50) == 0) { lean_object* x_51; lean_object* x_52; @@ -114388,8 +113270,8 @@ lean_dec(x_51); x_12 = x_52; x_13 = x_42; x_14 = x_43; -x_15 = x_45; -x_16 = x_44; +x_15 = x_44; +x_16 = x_45; x_17 = lean_box(0); goto block_39; } @@ -114422,23 +113304,23 @@ goto block_39; } else { -x_40 = x_54; -x_41 = lean_box(0); +x_40 = lean_box(0); +x_41 = x_54; x_42 = x_55; x_43 = x_56; -x_44 = x_58; -x_45 = x_57; +x_44 = x_57; +x_45 = x_58; goto block_53; } } else { -x_40 = x_54; -x_41 = lean_box(0); +x_40 = lean_box(0); +x_41 = x_54; x_42 = x_55; x_43 = x_56; -x_44 = x_58; -x_45 = x_57; +x_44 = x_57; +x_45 = x_58; goto block_53; } } @@ -120269,22 +119151,22 @@ l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_Fu lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__5); l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__6 = _init_l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__6(); lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__13___redArg___closed__6); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__0); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__1); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__2); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__2___closed__3); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__0); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__1); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__2); -l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3(); -lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17_spec__31___lam__0___closed__3); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__0); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__1); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__2); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__2___closed__3); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__0); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__1); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__2); +l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3 = _init_l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3(); +lean_mark_persistent(l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize_spec__17___redArg___lam__3___closed__3); l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__1___closed__0 = _init_l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__1___closed__0(); lean_mark_persistent(l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__1___closed__0); l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__1___closed__1 = _init_l___private_Lean_Meta_Tactic_FunInd_0__Lean_Tactic_FunInd_deriveInductionStructural_doRealize___lam__1___closed__1(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/AC/Eq.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/AC/Eq.c index 2ba0673d6018..59ff841cb378 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/AC/Eq.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/AC/Eq.c @@ -21949,9 +21949,9 @@ goto block_154; block_147: { lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_144 = lean_nat_add(x_142, x_143); +x_144 = lean_nat_add(x_141, x_143); lean_dec(x_143); -lean_dec(x_142); +lean_dec(x_141); if (lean_is_scalar(x_138)) { x_145 = lean_alloc_ctor(0, 5, 0); } else { @@ -21970,7 +21970,7 @@ if (lean_is_scalar(x_128)) { lean_ctor_set(x_146, 0, x_140); lean_ctor_set(x_146, 1, x_130); lean_ctor_set(x_146, 2, x_131); -lean_ctor_set(x_146, 3, x_141); +lean_ctor_set(x_146, 3, x_142); lean_ctor_set(x_146, 4, x_145); return x_146; } @@ -21996,8 +21996,8 @@ if (lean_obj_tag(x_133) == 0) lean_object* x_152; x_152 = lean_ctor_get(x_133, 0); lean_inc(x_152); -x_141 = x_150; -x_142 = x_151; +x_141 = x_151; +x_142 = x_150; x_143 = x_152; goto block_147; } @@ -22005,8 +22005,8 @@ else { lean_object* x_153; x_153 = lean_unsigned_to_nat(0u); -x_141 = x_150; -x_142 = x_151; +x_141 = x_151; +x_142 = x_150; x_143 = x_153; goto block_147; } @@ -23200,7 +23200,7 @@ return x_33; { lean_object* x_45; lean_object* x_46; x_45 = l_List_forIn_x27_loop___at___00List_forIn_x27_loop___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__3_spec__3___redArg___closed__3; -x_46 = l_panic___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__0(x_45, x_43, x_41, x_37, x_36, x_38, x_39, x_42, x_40, x_35); +x_46 = l_panic___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__0(x_45, x_39, x_44, x_42, x_38, x_43, x_41, x_36, x_35, x_37); x_20 = x_46; goto block_34; } @@ -23208,17 +23208,17 @@ goto block_34; { lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; x_67 = lean_ctor_get(x_3, 1); -lean_inc_ref(x_56); -lean_inc_ref(x_67); -x_68 = l_Lean_Grind_AC_Seq_union(x_67, x_56); lean_inc_ref(x_54); +lean_inc_ref(x_67); +x_68 = l_Lean_Grind_AC_Seq_union(x_67, x_54); +lean_inc_ref(x_55); lean_inc_ref(x_53); -x_69 = l_Lean_Grind_AC_Seq_union(x_53, x_54); +x_69 = l_Lean_Grind_AC_Seq_union(x_53, x_55); lean_inc_ref(x_3); x_70 = lean_alloc_ctor(9, 5, 0); -lean_ctor_set(x_70, 0, x_54); -lean_ctor_set(x_70, 1, x_55); -lean_ctor_set(x_70, 2, x_56); +lean_ctor_set(x_70, 0, x_55); +lean_ctor_set(x_70, 1, x_56); +lean_ctor_set(x_70, 2, x_54); lean_ctor_set(x_70, 3, x_3); lean_ctor_set(x_70, 4, x_17); lean_inc(x_57); @@ -23340,16 +23340,16 @@ if (x_91 == 0) if (x_89 == 0) { lean_dec(x_17); -x_35 = x_87; -x_36 = x_82; -x_37 = x_81; -x_38 = x_83; -x_39 = x_84; -x_40 = x_86; -x_41 = x_80; -x_42 = x_85; -x_43 = x_79; -x_44 = lean_box(0); +x_35 = x_86; +x_36 = x_85; +x_37 = x_87; +x_38 = x_82; +x_39 = x_79; +x_40 = lean_box(0); +x_41 = x_84; +x_42 = x_81; +x_43 = x_83; +x_44 = x_80; goto block_47; } else @@ -23379,9 +23379,9 @@ x_99 = l_List_forIn_x27_loop___at___00List_forIn_x27_loop___at___00__private_Lea x_100 = l_Lean_Option_get___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__1(x_98, x_99); if (x_100 == 0) { -x_54 = x_95; -x_55 = x_96; -x_56 = x_97; +x_54 = x_97; +x_55 = x_95; +x_56 = x_96; x_57 = x_79; x_58 = x_80; x_59 = x_81; @@ -23436,9 +23436,9 @@ goto block_34; } else { -x_54 = x_95; -x_55 = x_96; -x_56 = x_97; +x_54 = x_97; +x_55 = x_95; +x_56 = x_96; x_57 = x_79; x_58 = x_80; x_59 = x_81; @@ -23494,16 +23494,16 @@ return x_110; else { lean_dec(x_17); -x_35 = x_87; -x_36 = x_82; -x_37 = x_81; -x_38 = x_83; -x_39 = x_84; -x_40 = x_86; -x_41 = x_80; -x_42 = x_85; -x_43 = x_79; -x_44 = lean_box(0); +x_35 = x_86; +x_36 = x_85; +x_37 = x_87; +x_38 = x_82; +x_39 = x_79; +x_40 = lean_box(0); +x_41 = x_84; +x_42 = x_81; +x_43 = x_83; +x_44 = x_80; goto block_47; } } @@ -23895,7 +23895,7 @@ return x_34; { lean_object* x_46; lean_object* x_47; x_46 = l_List_forIn_x27_loop___at___00List_forIn_x27_loop___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__3_spec__3___redArg___closed__3; -x_47 = l_panic___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__0(x_46, x_37, x_45, x_40, x_44, x_36, x_39, x_43, x_42, x_38); +x_47 = l_panic___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_EqCnstr_superposeWithAC_spec__0(x_46, x_43, x_40, x_38, x_37, x_39, x_45, x_42, x_44, x_36); x_21 = x_47; goto block_35; } @@ -24027,16 +24027,16 @@ if (x_92 == 0) if (x_90 == 0) { lean_dec(x_18); -x_36 = x_84; -x_37 = x_80; -x_38 = x_88; -x_39 = x_85; -x_40 = x_82; +x_36 = x_88; +x_37 = x_83; +x_38 = x_82; +x_39 = x_84; +x_40 = x_81; x_41 = lean_box(0); -x_42 = x_87; -x_43 = x_86; -x_44 = x_83; -x_45 = x_81; +x_42 = x_86; +x_43 = x_80; +x_44 = x_87; +x_45 = x_85; goto block_48; } else @@ -24177,16 +24177,16 @@ return x_111; else { lean_dec(x_18); -x_36 = x_84; -x_37 = x_80; -x_38 = x_88; -x_39 = x_85; -x_40 = x_82; +x_36 = x_88; +x_37 = x_83; +x_38 = x_82; +x_39 = x_84; +x_40 = x_81; x_41 = lean_box(0); -x_42 = x_87; -x_43 = x_86; -x_44 = x_83; -x_45 = x_81; +x_42 = x_86; +x_43 = x_80; +x_44 = x_87; +x_45 = x_85; goto block_48; } } @@ -28995,9 +28995,9 @@ goto block_49; block_42: { lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_nat_add(x_37, x_38); +x_39 = lean_nat_add(x_36, x_38); lean_dec(x_38); -lean_dec(x_37); +lean_dec(x_36); if (lean_is_scalar(x_33)) { x_40 = lean_alloc_ctor(0, 5, 0); } else { @@ -29016,7 +29016,7 @@ if (lean_is_scalar(x_23)) { lean_ctor_set(x_41, 0, x_35); lean_ctor_set(x_41, 1, x_25); lean_ctor_set(x_41, 2, x_26); -lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 3, x_37); lean_ctor_set(x_41, 4, x_40); return x_41; } @@ -29042,8 +29042,8 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_47; x_47 = lean_ctor_get(x_28, 0); lean_inc(x_47); -x_36 = x_45; -x_37 = x_46; +x_36 = x_46; +x_37 = x_45; x_38 = x_47; goto block_42; } @@ -29051,8 +29051,8 @@ else { lean_object* x_48; x_48 = lean_unsigned_to_nat(0u); -x_36 = x_45; -x_37 = x_46; +x_36 = x_46; +x_37 = x_45; x_38 = x_48; goto block_42; } @@ -30876,9 +30876,9 @@ goto block_454; block_446: { lean_object* x_443; lean_object* x_444; lean_object* x_445; -x_443 = lean_nat_add(x_441, x_442); +x_443 = lean_nat_add(x_440, x_442); lean_dec(x_442); -lean_dec(x_441); +lean_dec(x_440); if (lean_is_scalar(x_437)) { x_444 = lean_alloc_ctor(0, 5, 0); } else { @@ -30897,7 +30897,7 @@ if (lean_is_scalar(x_427)) { lean_ctor_set(x_445, 0, x_439); lean_ctor_set(x_445, 1, x_430); lean_ctor_set(x_445, 2, x_431); -lean_ctor_set(x_445, 3, x_440); +lean_ctor_set(x_445, 3, x_441); lean_ctor_set(x_445, 4, x_444); return x_445; } @@ -30924,8 +30924,8 @@ if (lean_obj_tag(x_433) == 0) lean_object* x_452; x_452 = lean_ctor_get(x_433, 0); lean_inc(x_452); -x_440 = x_450; -x_441 = x_451; +x_440 = x_451; +x_441 = x_450; x_442 = x_452; goto block_446; } @@ -30933,8 +30933,8 @@ else { lean_object* x_453; x_453 = lean_unsigned_to_nat(0u); -x_440 = x_450; -x_441 = x_451; +x_440 = x_451; +x_441 = x_450; x_442 = x_453; goto block_446; } @@ -37622,11 +37622,11 @@ x_117 = l_List_forIn_x27_loop___at___00List_forIn_x27_loop___at___00__private_Le x_118 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_118, 0, x_116); lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_MessageData_ofExpr(x_99); +x_119 = l_Lean_MessageData_ofExpr(x_104); 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_addTrace___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_propagateEqs_process_spec__2___redArg(x_16, x_120, x_108, x_95, x_104, x_98, x_101); +x_121 = l_Lean_addTrace___at___00__private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC_propagateEqs_process_spec__2___redArg(x_16, x_120, x_108, x_106, x_102, x_95, x_107); if (lean_obj_tag(x_121) == 0) { lean_object* x_122; lean_object* x_123; @@ -37636,31 +37636,31 @@ lean_dec_ref(x_121); x_123 = lean_ctor_get(x_122, 1); lean_inc(x_123); lean_dec(x_122); -x_26 = x_100; +x_26 = x_99; x_27 = x_123; -x_28 = x_103; -x_29 = x_106; -x_30 = x_102; -x_31 = x_96; -x_32 = x_107; -x_33 = x_95; -x_34 = x_104; -x_35 = x_98; -x_36 = x_101; +x_28 = x_96; +x_29 = x_98; +x_30 = x_101; +x_31 = x_105; +x_32 = x_103; +x_33 = x_106; +x_34 = x_102; +x_35 = x_95; +x_36 = x_107; x_37 = lean_box(0); goto block_94; } else { lean_dec(x_107); -lean_dec(x_106); -lean_dec(x_104); +lean_dec_ref(x_106); +lean_dec_ref(x_105); lean_dec(x_103); lean_dec(x_102); lean_dec(x_101); -lean_dec_ref(x_100); -lean_dec_ref(x_98); -lean_dec_ref(x_96); +lean_dec_ref(x_99); +lean_dec(x_98); +lean_dec(x_96); lean_dec_ref(x_95); lean_dec_ref(x_25); lean_dec_ref(x_24); @@ -37734,19 +37734,19 @@ if (x_151 == 0) { lean_object* x_152; x_152 = l___private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC___aux__Lean__Meta__Tactic__Grind__AC__Eq______macroRules____private__Lean__Meta__Tactic__Grind__AC__Eq__0__Lean__Meta__Grind__AC__commandGen__cnstr__fns____1___closed__253; -x_95 = x_132; -x_96 = x_130; +x_95 = x_134; +x_96 = x_127; x_97 = x_150; -x_98 = x_134; -x_99 = x_147; -x_100 = x_140; -x_101 = x_135; -x_102 = x_129; -x_103 = x_127; -x_104 = x_133; -x_105 = lean_box(0); -x_106 = x_128; -x_107 = x_131; +x_98 = x_128; +x_99 = x_140; +x_100 = lean_box(0); +x_101 = x_129; +x_102 = x_133; +x_103 = x_131; +x_104 = x_147; +x_105 = x_130; +x_106 = x_132; +x_107 = x_135; x_108 = x_146; x_109 = x_152; goto block_124; @@ -37755,19 +37755,19 @@ else { lean_object* x_153; x_153 = l___private_Lean_Meta_Tactic_Grind_AC_Eq_0__Lean_Meta_Grind_AC___aux__Lean__Meta__Tactic__Grind__AC__Eq______macroRules____private__Lean__Meta__Tactic__Grind__AC__Eq__0__Lean__Meta__Grind__AC__commandGen__cnstr__fns____1___closed__220; -x_95 = x_132; -x_96 = x_130; +x_95 = x_134; +x_96 = x_127; x_97 = x_150; -x_98 = x_134; -x_99 = x_147; -x_100 = x_140; -x_101 = x_135; -x_102 = x_129; -x_103 = x_127; -x_104 = x_133; -x_105 = lean_box(0); -x_106 = x_128; -x_107 = x_131; +x_98 = x_128; +x_99 = x_140; +x_100 = lean_box(0); +x_101 = x_129; +x_102 = x_133; +x_103 = x_131; +x_104 = x_147; +x_105 = x_130; +x_106 = x_132; +x_107 = x_135; x_108 = x_146; x_109 = x_153; goto block_124; diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c index 4e070f5bd28d..10e19b7cdbf2 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c @@ -16173,45 +16173,45 @@ return x_203; block_112: { lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Meta_Context_config(x_25); +x_30 = l_Lean_Meta_Context_config(x_28); x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) { uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; uint8_t x_40; uint64_t x_41; uint8_t x_42; -x_32 = lean_ctor_get_uint8(x_25, sizeof(void*)*7); -x_33 = lean_ctor_get(x_25, 1); +x_32 = lean_ctor_get_uint8(x_28, sizeof(void*)*7); +x_33 = lean_ctor_get(x_28, 1); lean_inc(x_33); -x_34 = lean_ctor_get(x_25, 2); +x_34 = lean_ctor_get(x_28, 2); lean_inc_ref(x_34); -x_35 = lean_ctor_get(x_25, 3); +x_35 = lean_ctor_get(x_28, 3); lean_inc_ref(x_35); -x_36 = lean_ctor_get(x_25, 4); +x_36 = lean_ctor_get(x_28, 4); lean_inc(x_36); -x_37 = lean_ctor_get(x_25, 5); +x_37 = lean_ctor_get(x_28, 5); lean_inc(x_37); -x_38 = lean_ctor_get(x_25, 6); +x_38 = lean_ctor_get(x_28, 6); lean_inc(x_38); -x_39 = lean_ctor_get_uint8(x_25, sizeof(void*)*7 + 1); -x_40 = lean_ctor_get_uint8(x_25, sizeof(void*)*7 + 2); +x_39 = lean_ctor_get_uint8(x_28, sizeof(void*)*7 + 1); +x_40 = lean_ctor_get_uint8(x_28, sizeof(void*)*7 + 2); lean_ctor_set_uint8(x_30, 9, x_29); -x_41 = l_Lean_Meta_Context_configKey(x_25); -x_42 = !lean_is_exclusive(x_25); +x_41 = l_Lean_Meta_Context_configKey(x_28); +x_42 = !lean_is_exclusive(x_28); if (x_42 == 0) { lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; lean_object* x_55; lean_object* x_56; -x_43 = lean_ctor_get(x_25, 6); +x_43 = lean_ctor_get(x_28, 6); lean_dec(x_43); -x_44 = lean_ctor_get(x_25, 5); +x_44 = lean_ctor_get(x_28, 5); lean_dec(x_44); -x_45 = lean_ctor_get(x_25, 4); +x_45 = lean_ctor_get(x_28, 4); lean_dec(x_45); -x_46 = lean_ctor_get(x_25, 3); +x_46 = lean_ctor_get(x_28, 3); lean_dec(x_46); -x_47 = lean_ctor_get(x_25, 2); +x_47 = lean_ctor_get(x_28, 2); lean_dec(x_47); -x_48 = lean_ctor_get(x_25, 1); +x_48 = lean_ctor_get(x_28, 1); lean_dec(x_48); -x_49 = lean_ctor_get(x_25, 0); +x_49 = lean_ctor_get(x_28, 0); lean_dec(x_49); x_50 = 2; x_51 = lean_uint64_shift_right(x_41, x_50); @@ -16221,8 +16221,8 @@ x_54 = lean_uint64_lor(x_52, x_53); x_55 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_55, 0, x_30); lean_ctor_set_uint64(x_55, sizeof(void*)*1, x_54); -lean_ctor_set(x_25, 0, x_55); -x_56 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_20, x_28, x_18, x_3, x_21, x_27, x_24, x_19, x_25, x_26, x_23, x_17); +lean_ctor_set(x_28, 0, x_55); +x_56 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_18, x_27, x_23, x_3, x_22, x_17, x_21, x_26, x_28, x_25, x_24, x_20); if (lean_obj_tag(x_56) == 0) { uint8_t x_57; @@ -16250,7 +16250,7 @@ return x_56; else { uint64_t x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_25); +lean_dec(x_28); x_60 = 2; x_61 = lean_uint64_shift_right(x_41, x_60); x_62 = lean_uint64_shift_left(x_61, x_60); @@ -16270,7 +16270,7 @@ lean_ctor_set(x_66, 6, x_38); lean_ctor_set_uint8(x_66, sizeof(void*)*7, x_32); lean_ctor_set_uint8(x_66, sizeof(void*)*7 + 1, x_39); lean_ctor_set_uint8(x_66, sizeof(void*)*7 + 2, x_40); -x_67 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_20, x_28, x_18, x_3, x_21, x_27, x_24, x_19, x_66, x_26, x_23, x_17); +x_67 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_18, x_27, x_23, x_3, x_22, x_17, x_21, x_26, x_66, x_25, x_24, x_20); if (lean_obj_tag(x_67) == 0) { lean_object* x_68; lean_object* x_69; lean_object* x_70; @@ -16319,21 +16319,21 @@ x_86 = lean_ctor_get_uint8(x_30, 16); x_87 = lean_ctor_get_uint8(x_30, 17); x_88 = lean_ctor_get_uint8(x_30, 18); lean_dec(x_30); -x_89 = lean_ctor_get_uint8(x_25, sizeof(void*)*7); -x_90 = lean_ctor_get(x_25, 1); +x_89 = lean_ctor_get_uint8(x_28, sizeof(void*)*7); +x_90 = lean_ctor_get(x_28, 1); lean_inc(x_90); -x_91 = lean_ctor_get(x_25, 2); +x_91 = lean_ctor_get(x_28, 2); lean_inc_ref(x_91); -x_92 = lean_ctor_get(x_25, 3); +x_92 = lean_ctor_get(x_28, 3); lean_inc_ref(x_92); -x_93 = lean_ctor_get(x_25, 4); +x_93 = lean_ctor_get(x_28, 4); lean_inc(x_93); -x_94 = lean_ctor_get(x_25, 5); +x_94 = lean_ctor_get(x_28, 5); lean_inc(x_94); -x_95 = lean_ctor_get(x_25, 6); +x_95 = lean_ctor_get(x_28, 6); lean_inc(x_95); -x_96 = lean_ctor_get_uint8(x_25, sizeof(void*)*7 + 1); -x_97 = lean_ctor_get_uint8(x_25, sizeof(void*)*7 + 2); +x_96 = lean_ctor_get_uint8(x_28, sizeof(void*)*7 + 1); +x_97 = lean_ctor_get_uint8(x_28, sizeof(void*)*7 + 2); x_98 = lean_alloc_ctor(0, 0, 19); lean_ctor_set_uint8(x_98, 0, x_71); lean_ctor_set_uint8(x_98, 1, x_72); @@ -16354,18 +16354,18 @@ lean_ctor_set_uint8(x_98, 15, x_85); lean_ctor_set_uint8(x_98, 16, x_86); lean_ctor_set_uint8(x_98, 17, x_87); lean_ctor_set_uint8(x_98, 18, x_88); -x_99 = l_Lean_Meta_Context_configKey(x_25); -if (lean_is_exclusive(x_25)) { - lean_ctor_release(x_25, 0); - lean_ctor_release(x_25, 1); - lean_ctor_release(x_25, 2); - lean_ctor_release(x_25, 3); - lean_ctor_release(x_25, 4); - lean_ctor_release(x_25, 5); - lean_ctor_release(x_25, 6); - x_100 = x_25; +x_99 = l_Lean_Meta_Context_configKey(x_28); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + lean_ctor_release(x_28, 2); + lean_ctor_release(x_28, 3); + lean_ctor_release(x_28, 4); + lean_ctor_release(x_28, 5); + lean_ctor_release(x_28, 6); + x_100 = x_28; } else { - lean_dec_ref(x_25); + lean_dec_ref(x_28); x_100 = lean_box(0); } x_101 = 2; @@ -16391,7 +16391,7 @@ lean_ctor_set(x_107, 6, x_95); lean_ctor_set_uint8(x_107, sizeof(void*)*7, x_89); lean_ctor_set_uint8(x_107, sizeof(void*)*7 + 1, x_96); lean_ctor_set_uint8(x_107, sizeof(void*)*7 + 2, x_97); -x_108 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_20, x_28, x_18, x_3, x_21, x_27, x_24, x_19, x_107, x_26, x_23, x_17); +x_108 = l_Lean_Meta_Grind_addTheoremInstance(x_1, x_18, x_27, x_23, x_3, x_22, x_17, x_21, x_26, x_107, x_25, x_24, x_20); if (lean_obj_tag(x_108) == 0) { lean_object* x_109; lean_object* x_110; lean_object* x_111; @@ -16436,18 +16436,18 @@ if (x_126 == 0) { uint8_t x_129; x_129 = 1; -x_17 = x_122; -x_18 = x_128; -x_19 = x_118; -x_20 = x_113; -x_21 = x_115; -x_22 = lean_box(0); -x_23 = x_121; -x_24 = x_117; -x_25 = x_119; -x_26 = x_120; -x_27 = x_116; -x_28 = x_114; +x_17 = x_116; +x_18 = x_113; +x_19 = lean_box(0); +x_20 = x_122; +x_21 = x_117; +x_22 = x_115; +x_23 = x_128; +x_24 = x_121; +x_25 = x_120; +x_26 = x_118; +x_27 = x_114; +x_28 = x_119; x_29 = x_129; goto block_112; } @@ -16455,18 +16455,18 @@ else { uint8_t x_130; x_130 = 2; -x_17 = x_122; -x_18 = x_128; -x_19 = x_118; -x_20 = x_113; -x_21 = x_115; -x_22 = lean_box(0); -x_23 = x_121; -x_24 = x_117; -x_25 = x_119; -x_26 = x_120; -x_27 = x_116; -x_28 = x_114; +x_17 = x_116; +x_18 = x_113; +x_19 = lean_box(0); +x_20 = x_122; +x_21 = x_117; +x_22 = x_115; +x_23 = x_128; +x_24 = x_121; +x_25 = x_120; +x_26 = x_118; +x_27 = x_114; +x_28 = x_119; x_29 = x_130; goto block_112; } @@ -27873,10 +27873,10 @@ x_83 = l_Lean_Expr_isLambda(x_1); if (x_83 == 0) { x_68 = x_81; -x_69 = x_82; -x_70 = lean_box(0); -x_71 = x_80; -x_72 = x_79; +x_69 = x_80; +x_70 = x_79; +x_71 = lean_box(0); +x_72 = x_82; x_73 = x_83; goto block_76; } @@ -27885,20 +27885,20 @@ else if (x_2 == 0) { x_68 = x_81; -x_69 = x_82; -x_70 = lean_box(0); -x_71 = x_80; -x_72 = x_79; +x_69 = x_80; +x_70 = x_79; +x_71 = lean_box(0); +x_72 = x_82; x_73 = x_83; goto block_76; } else { -x_8 = x_82; -x_9 = x_81; -x_10 = lean_box(0); -x_11 = x_80; -x_12 = x_79; +x_8 = x_81; +x_9 = x_80; +x_10 = x_79; +x_11 = lean_box(0); +x_12 = x_82; goto block_67; } } @@ -27931,12 +27931,12 @@ return x_128; block_67: { lean_object* x_13; -lean_inc(x_8); -lean_inc_ref(x_9); -lean_inc(x_11); -lean_inc_ref(x_12); +lean_inc(x_12); +lean_inc_ref(x_8); +lean_inc(x_9); +lean_inc_ref(x_10); lean_inc_ref(x_1); -x_13 = l_Lean_Meta_isLitValue(x_1, x_12, x_11, x_9, x_8); +x_13 = l_Lean_Meta_isLitValue(x_1, x_10, x_9, x_8, x_12); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; uint8_t x_15; @@ -27947,11 +27947,11 @@ if (x_15 == 0) { lean_object* x_16; lean_dec_ref(x_13); -lean_inc(x_8); -lean_inc_ref(x_9); -lean_inc(x_11); -lean_inc_ref(x_12); -x_16 = l_Lean_Meta_constructorApp_x27_x3f(x_1, x_12, x_11, x_9, x_8); +lean_inc(x_12); +lean_inc_ref(x_8); +lean_inc(x_9); +lean_inc_ref(x_10); +x_16 = l_Lean_Meta_constructorApp_x27_x3f(x_1, x_10, x_9, x_8, x_12); if (lean_obj_tag(x_16) == 0) { uint8_t x_17; @@ -27979,7 +27979,7 @@ lean_dec(x_20); x_23 = lean_array_get_size(x_21); x_24 = lean_box(0); x_25 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue___closed__0; -x_26 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue_spec__0___redArg(x_23, x_21, x_2, x_24, x_25, x_22, x_25, x_12, x_11, x_9, x_8); +x_26 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue_spec__0___redArg(x_23, x_21, x_2, x_24, x_25, x_22, x_25, x_10, x_9, x_8, x_12); lean_dec(x_21); if (lean_obj_tag(x_26) == 0) { @@ -28063,10 +28063,10 @@ return x_42; else { lean_dec(x_18); -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_12); +lean_dec_ref(x_10); +lean_dec(x_9); +lean_dec_ref(x_8); lean_ctor_set(x_16, 0, x_14); return x_16; } @@ -28095,7 +28095,7 @@ lean_dec(x_45); x_48 = lean_array_get_size(x_46); x_49 = lean_box(0); x_50 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue___closed__0; -x_51 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue_spec__0___redArg(x_48, x_46, x_2, x_49, x_50, x_47, x_50, x_12, x_11, x_9, x_8); +x_51 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_isValue_spec__0___redArg(x_48, x_46, x_2, x_49, x_50, x_47, x_50, x_10, x_9, x_8, x_12); lean_dec(x_46); if (lean_obj_tag(x_51) == 0) { @@ -28165,10 +28165,10 @@ else { lean_object* x_63; lean_dec(x_43); -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_12); +lean_dec_ref(x_10); +lean_dec(x_9); +lean_dec_ref(x_8); x_63 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_63, 0, x_14); return x_63; @@ -28179,10 +28179,10 @@ else { uint8_t x_64; lean_dec(x_14); -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_12); +lean_dec_ref(x_10); +lean_dec(x_9); +lean_dec_ref(x_8); x_64 = !lean_is_exclusive(x_16); if (x_64 == 0) { @@ -28203,20 +28203,20 @@ return x_66; else { lean_dec(x_14); -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_12); +lean_dec_ref(x_10); +lean_dec(x_9); +lean_dec_ref(x_8); lean_dec_ref(x_1); return x_13; } } else { -lean_dec_ref(x_12); -lean_dec(x_11); -lean_dec_ref(x_9); -lean_dec(x_8); +lean_dec(x_12); +lean_dec_ref(x_10); +lean_dec(x_9); +lean_dec_ref(x_8); lean_dec_ref(x_1); return x_13; } @@ -28225,18 +28225,18 @@ return x_13; { if (x_73 == 0) { -x_8 = x_69; -x_9 = x_68; -x_10 = lean_box(0); -x_11 = x_71; +x_8 = x_68; +x_9 = x_69; +x_10 = x_70; +x_11 = lean_box(0); x_12 = x_72; goto block_67; } else { lean_object* x_74; lean_object* x_75; -lean_dec_ref(x_72); -lean_dec(x_71); +lean_dec(x_72); +lean_dec_ref(x_70); lean_dec(x_69); lean_dec_ref(x_68); lean_dec_ref(x_1); @@ -32714,7 +32714,7 @@ lean_inc_ref(x_21); x_48 = l_Lean_Meta_Grind_markTheoremInstance___redArg(x_21, x_24, x_4); if (lean_obj_tag(x_48) == 0) { -lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_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_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; uint8_t x_190; 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; uint8_t x_286; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t 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_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_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_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_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; uint8_t x_190; 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; uint8_t x_286; x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); lean_dec_ref(x_48); @@ -32846,7 +32846,7 @@ goto block_47; block_75: { lean_object* x_66; lean_object* x_67; uint8_t x_68; uint8_t x_69; uint8_t x_70; lean_object* x_71; -x_66 = l_Lean_instantiateMVars___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__0___redArg(x_54, x_62); +x_66 = l_Lean_instantiateMVars___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__0___redArg(x_50, x_62); x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); lean_dec_ref(x_66); @@ -32854,16 +32854,16 @@ x_68 = 0; x_69 = lean_unbox(x_49); x_70 = lean_unbox(x_49); lean_dec(x_49); -x_71 = l_Lean_Meta_mkLambdaFVars(x_51, x_67, x_50, x_69, x_50, x_70, x_68, x_61, x_62, x_63, x_64); -lean_dec_ref(x_51); +x_71 = l_Lean_Meta_mkLambdaFVars(x_54, x_67, x_53, x_69, x_53, x_70, x_68, x_61, x_62, x_63, x_64); +lean_dec_ref(x_54); if (lean_obj_tag(x_71) == 0) { lean_object* x_72; lean_object* x_73; x_72 = lean_ctor_get(x_71, 0); lean_inc(x_72); lean_dec_ref(x_71); -x_73 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_19, x_72, x_53, x_52, x_55, x_56, x_57, x_58, x_59, x_60, x_61, x_62, x_63, x_64); -lean_dec(x_53); +x_73 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_19, x_72, x_51, x_52, x_55, x_56, x_57, x_58, x_59, x_60, x_61, x_62, x_63, x_64); +lean_dec(x_51); x_44 = x_73; goto block_47; } @@ -32880,8 +32880,8 @@ lean_dec(x_58); lean_dec(x_57); lean_dec(x_56); lean_dec_ref(x_55); -lean_dec(x_53); lean_dec(x_52); +lean_dec(x_51); lean_dec_ref(x_19); x_74 = lean_ctor_get(x_71, 0); lean_inc(x_74); @@ -32898,11 +32898,11 @@ x_92 = lean_box(0); x_93 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__2___closed__0; x_94 = lean_array_size(x_90); x_95 = 0; -lean_inc(x_76); -lean_inc_ref(x_87); -lean_inc(x_86); +lean_inc(x_85); lean_inc_ref(x_80); -x_96 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__2___redArg(x_93, x_92, x_90, x_94, x_95, x_93, x_80, x_86, x_87, x_76); +lean_inc(x_87); +lean_inc_ref(x_79); +x_96 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__2___redArg(x_93, x_92, x_90, x_94, x_95, x_93, x_79, x_87, x_80, x_85); if (lean_obj_tag(x_96) == 0) { lean_object* x_97; uint8_t x_98; @@ -32919,21 +32919,21 @@ lean_dec(x_100); if (lean_obj_tag(x_99) == 0) { lean_free_object(x_97); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -32949,7 +32949,7 @@ lean_object* x_102; lean_object* x_103; x_102 = lean_ctor_get(x_101, 0); lean_inc(x_102); lean_dec_ref(x_101); -x_103 = l_Lean_Meta_Grind_getConfig___redArg(x_79); +x_103 = l_Lean_Meta_Grind_getConfig___redArg(x_88); if (lean_obj_tag(x_103) == 0) { lean_object* x_104; uint8_t x_105; @@ -32962,60 +32962,60 @@ if (x_105 == 0) { lean_dec(x_102); lean_free_object(x_97); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } else { lean_object* x_106; lean_object* x_107; uint8_t x_108; -x_106 = lean_ctor_get(x_87, 2); +x_106 = lean_ctor_get(x_80, 2); x_107 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___closed__0; x_108 = l_Lean_Option_get___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__2(x_106, x_107); if (x_108 == 0) { lean_dec(x_102); lean_free_object(x_97); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } else { lean_object* x_109; -lean_inc(x_76); -lean_inc_ref(x_87); -lean_inc(x_86); +lean_inc(x_85); lean_inc_ref(x_80); -x_109 = lean_infer_type(x_102, x_80, x_86, x_87, x_76); +lean_inc(x_87); +lean_inc_ref(x_79); +x_109 = lean_infer_type(x_102, x_79, x_87, x_80, x_85); if (lean_obj_tag(x_109) == 0) { lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; @@ -33036,25 +33036,25 @@ x_115 = l_Lean_indentExpr(x_110); 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_Meta_Grind_reportIssue(x_116, x_85, x_79, x_81, x_80, x_86, x_87, x_76); +x_117 = l_Lean_Meta_Grind_reportIssue(x_116, x_86, x_88, x_83, x_79, x_87, x_80, x_85); if (lean_obj_tag(x_117) == 0) { lean_dec_ref(x_117); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -33062,18 +33062,18 @@ else { lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_44 = x_117; @@ -33086,18 +33086,18 @@ lean_object* x_118; lean_free_object(x_97); lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_118 = lean_ctor_get(x_109, 0); @@ -33117,18 +33117,18 @@ lean_dec(x_102); lean_free_object(x_97); lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_119 = lean_ctor_get(x_103, 0); @@ -33143,21 +33143,21 @@ else { lean_dec(x_101); lean_free_object(x_97); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -33171,21 +33171,21 @@ lean_inc(x_120); lean_dec(x_97); if (lean_obj_tag(x_120) == 0) { -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -33201,7 +33201,7 @@ lean_object* x_122; lean_object* x_123; x_122 = lean_ctor_get(x_121, 0); lean_inc(x_122); lean_dec_ref(x_121); -x_123 = l_Lean_Meta_Grind_getConfig___redArg(x_79); +x_123 = l_Lean_Meta_Grind_getConfig___redArg(x_88); if (lean_obj_tag(x_123) == 0) { lean_object* x_124; uint8_t x_125; @@ -33213,59 +33213,59 @@ lean_dec(x_124); if (x_125 == 0) { lean_dec(x_122); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } else { lean_object* x_126; lean_object* x_127; uint8_t x_128; -x_126 = lean_ctor_get(x_87, 2); +x_126 = lean_ctor_get(x_80, 2); x_127 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___closed__0; x_128 = l_Lean_Option_get___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__2(x_126, x_127); if (x_128 == 0) { lean_dec(x_122); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } else { lean_object* x_129; -lean_inc(x_76); -lean_inc_ref(x_87); -lean_inc(x_86); +lean_inc(x_85); lean_inc_ref(x_80); -x_129 = lean_infer_type(x_122, x_80, x_86, x_87, x_76); +lean_inc(x_87); +lean_inc_ref(x_79); +x_129 = lean_infer_type(x_122, x_79, x_87, x_80, x_85); if (lean_obj_tag(x_129) == 0) { lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; @@ -33286,25 +33286,25 @@ x_136 = l_Lean_indentExpr(x_130); x_137 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_137, 0, x_135); lean_ctor_set(x_137, 1, x_136); -x_138 = l_Lean_Meta_Grind_reportIssue(x_137, x_85, x_79, x_81, x_80, x_86, x_87, x_76); +x_138 = l_Lean_Meta_Grind_reportIssue(x_137, x_86, x_88, x_83, x_79, x_87, x_80, x_85); if (lean_obj_tag(x_138) == 0) { lean_dec_ref(x_138); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -33312,18 +33312,18 @@ else { lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_44 = x_138; @@ -33335,18 +33335,18 @@ else lean_object* x_139; lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_139 = lean_ctor_get(x_129, 0); @@ -33365,18 +33365,18 @@ lean_object* x_140; lean_dec(x_122); lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_140 = lean_ctor_get(x_123, 0); @@ -33390,21 +33390,21 @@ goto block_32; else { lean_dec(x_121); -x_50 = x_77; -x_51 = x_90; -x_52 = x_83; -x_53 = x_88; -x_54 = x_84; -x_55 = x_78; -x_56 = x_82; -x_57 = x_89; -x_58 = x_85; -x_59 = x_79; -x_60 = x_81; -x_61 = x_80; -x_62 = x_86; -x_63 = x_87; -x_64 = x_76; +x_50 = x_78; +x_51 = x_89; +x_52 = x_81; +x_53 = x_82; +x_54 = x_90; +x_55 = x_76; +x_56 = x_84; +x_57 = x_77; +x_58 = x_86; +x_59 = x_88; +x_60 = x_83; +x_61 = x_79; +x_62 = x_87; +x_63 = x_80; +x_64 = x_85; x_65 = lean_box(0); goto block_75; } @@ -33416,18 +33416,18 @@ else lean_object* x_141; lean_dec_ref(x_90); lean_dec(x_89); -lean_dec(x_88); -lean_dec_ref(x_87); +lean_dec_ref(x_88); +lean_dec(x_87); lean_dec(x_86); lean_dec(x_85); -lean_dec_ref(x_84); +lean_dec(x_84); lean_dec(x_83); -lean_dec(x_82); lean_dec(x_81); lean_dec_ref(x_80); lean_dec_ref(x_79); lean_dec_ref(x_78); -lean_dec(x_76); +lean_dec(x_77); +lean_dec_ref(x_76); lean_dec(x_49); lean_dec_ref(x_19); x_141 = lean_ctor_get(x_96, 0); @@ -33450,29 +33450,29 @@ x_161 = lean_unbox(x_160); if (x_161 == 0) { lean_object* x_162; uint8_t x_163; -x_162 = lean_mk_empty_array_with_capacity(x_153); -x_163 = lean_nat_dec_lt(x_153, x_158); +x_162 = lean_mk_empty_array_with_capacity(x_143); +x_163 = lean_nat_dec_lt(x_143, x_145); if (x_163 == 0) { uint8_t x_164; -lean_dec(x_158); -lean_dec_ref(x_155); +lean_dec_ref(x_157); +lean_dec(x_145); x_164 = lean_unbox(x_160); lean_dec(x_160); -x_76 = x_143; -x_77 = x_164; -x_78 = x_144; -x_79 = x_145; -x_80 = x_146; -x_81 = x_147; -x_82 = x_148; -x_83 = x_149; -x_84 = x_150; -x_85 = x_151; -x_86 = x_152; -x_87 = x_154; +x_76 = x_144; +x_77 = x_146; +x_78 = x_147; +x_79 = x_148; +x_80 = x_149; +x_81 = x_150; +x_82 = x_164; +x_83 = x_151; +x_84 = x_152; +x_85 = x_153; +x_86 = x_154; +x_87 = x_155; x_88 = x_156; -x_89 = x_157; +x_89 = x_158; x_90 = x_162; x_91 = lean_box(0); goto block_142; @@ -33480,28 +33480,28 @@ goto block_142; else { uint8_t x_165; -x_165 = lean_nat_dec_le(x_158, x_158); +x_165 = lean_nat_dec_le(x_145, x_145); if (x_165 == 0) { uint8_t x_166; -lean_dec(x_158); -lean_dec_ref(x_155); +lean_dec_ref(x_157); +lean_dec(x_145); x_166 = lean_unbox(x_160); lean_dec(x_160); -x_76 = x_143; -x_77 = x_166; -x_78 = x_144; -x_79 = x_145; -x_80 = x_146; -x_81 = x_147; -x_82 = x_148; -x_83 = x_149; -x_84 = x_150; -x_85 = x_151; -x_86 = x_152; -x_87 = x_154; +x_76 = x_144; +x_77 = x_146; +x_78 = x_147; +x_79 = x_148; +x_80 = x_149; +x_81 = x_150; +x_82 = x_166; +x_83 = x_151; +x_84 = x_152; +x_85 = x_153; +x_86 = x_154; +x_87 = x_155; x_88 = x_156; -x_89 = x_157; +x_89 = x_158; x_90 = x_162; x_91 = lean_box(0); goto block_142; @@ -33510,10 +33510,10 @@ else { size_t x_167; size_t x_168; lean_object* x_169; x_167 = 0; -x_168 = lean_usize_of_nat(x_158); -lean_dec(x_158); -x_169 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__3___redArg(x_155, x_167, x_168, x_162, x_144, x_148, x_157, x_151, x_145, x_147, x_146, x_152, x_154, x_143); -lean_dec_ref(x_155); +x_168 = lean_usize_of_nat(x_145); +lean_dec(x_145); +x_169 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__3___redArg(x_157, x_167, x_168, x_162, x_144, x_152, x_146, x_154, x_156, x_151, x_148, x_155, x_149, x_153); +lean_dec_ref(x_157); if (lean_obj_tag(x_169) == 0) { lean_object* x_170; uint8_t x_171; @@ -33522,20 +33522,20 @@ lean_inc(x_170); lean_dec_ref(x_169); x_171 = lean_unbox(x_160); lean_dec(x_160); -x_76 = x_143; -x_77 = x_171; -x_78 = x_144; -x_79 = x_145; -x_80 = x_146; -x_81 = x_147; -x_82 = x_148; -x_83 = x_149; -x_84 = x_150; -x_85 = x_151; -x_86 = x_152; -x_87 = x_154; +x_76 = x_144; +x_77 = x_146; +x_78 = x_147; +x_79 = x_148; +x_80 = x_149; +x_81 = x_150; +x_82 = x_171; +x_83 = x_151; +x_84 = x_152; +x_85 = x_153; +x_86 = x_154; +x_87 = x_155; x_88 = x_156; -x_89 = x_157; +x_89 = x_158; x_90 = x_170; x_91 = lean_box(0); goto block_142; @@ -33544,19 +33544,19 @@ else { lean_object* x_172; lean_dec(x_160); -lean_dec(x_157); -lean_dec(x_156); -lean_dec_ref(x_154); +lean_dec(x_158); +lean_dec_ref(x_156); +lean_dec(x_155); +lean_dec(x_154); +lean_dec(x_153); lean_dec(x_152); lean_dec(x_151); -lean_dec_ref(x_150); -lean_dec(x_149); -lean_dec(x_148); -lean_dec(x_147); -lean_dec_ref(x_146); -lean_dec_ref(x_145); +lean_dec(x_150); +lean_dec_ref(x_149); +lean_dec_ref(x_148); +lean_dec_ref(x_147); +lean_dec(x_146); lean_dec_ref(x_144); -lean_dec(x_143); lean_dec(x_49); lean_dec_ref(x_19); x_172 = lean_ctor_get(x_169, 0); @@ -33573,11 +33573,11 @@ else { lean_object* x_173; lean_dec(x_160); -lean_dec(x_158); -lean_dec_ref(x_155); +lean_dec_ref(x_157); +lean_dec(x_145); lean_dec(x_49); -x_173 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_19, x_150, x_156, x_149, x_144, x_148, x_157, x_151, x_145, x_147, x_146, x_152, x_154, x_143); -lean_dec(x_156); +x_173 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_19, x_147, x_158, x_150, x_144, x_152, x_146, x_154, x_156, x_151, x_148, x_155, x_149, x_153); +lean_dec(x_158); x_44 = x_173; goto block_47; } @@ -33586,20 +33586,20 @@ else { lean_object* x_174; lean_dec(x_158); -lean_dec(x_157); -lean_dec(x_156); -lean_dec_ref(x_155); -lean_dec_ref(x_154); +lean_dec_ref(x_157); +lean_dec_ref(x_156); +lean_dec(x_155); +lean_dec(x_154); +lean_dec(x_153); lean_dec(x_152); lean_dec(x_151); -lean_dec_ref(x_150); -lean_dec(x_149); -lean_dec(x_148); -lean_dec(x_147); -lean_dec_ref(x_146); -lean_dec_ref(x_145); +lean_dec(x_150); +lean_dec_ref(x_149); +lean_dec_ref(x_148); +lean_dec_ref(x_147); +lean_dec(x_146); +lean_dec(x_145); lean_dec_ref(x_144); -lean_dec(x_143); lean_dec(x_49); lean_dec_ref(x_19); x_174 = lean_ctor_get(x_159, 0); @@ -33613,17 +33613,17 @@ goto block_32; block_226: { lean_object* x_191; -lean_inc(x_176); -lean_inc_ref(x_187); -lean_inc(x_184); +lean_inc(x_182); lean_inc_ref(x_179); -lean_inc(x_181); +lean_inc(x_185); lean_inc_ref(x_178); -lean_inc(x_183); -lean_inc(x_189); -lean_inc(x_182); -lean_inc_ref(x_177); -x_191 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_applyAssignment(x_188, x_1, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); +lean_inc(x_180); +lean_inc_ref(x_188); +lean_inc(x_184); +lean_inc(x_177); +lean_inc(x_181); +lean_inc_ref(x_176); +x_191 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_applyAssignment(x_189, x_1, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); if (lean_obj_tag(x_191) == 0) { lean_object* x_192; lean_object* x_193; @@ -33637,12 +33637,12 @@ lean_object* x_194; lean_object* x_195; x_194 = lean_ctor_get(x_192, 1); lean_inc(x_194); lean_dec(x_192); -lean_inc(x_176); -lean_inc_ref(x_187); -lean_inc(x_184); +lean_inc(x_182); lean_inc_ref(x_179); -lean_inc_ref(x_177); -x_195 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_synthesizeInsts(x_188, x_180, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); +lean_inc(x_185); +lean_inc_ref(x_178); +lean_inc_ref(x_176); +x_195 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_synthesizeInsts(x_189, x_187, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); if (lean_obj_tag(x_195) == 0) { lean_object* x_196; @@ -33656,17 +33656,17 @@ lean_dec_ref(x_196); x_197 = lean_ctor_get(x_194, 1); lean_inc(x_197); lean_dec(x_194); -lean_inc(x_176); -lean_inc_ref(x_187); -lean_inc(x_184); +lean_inc(x_182); lean_inc_ref(x_179); -lean_inc(x_181); +lean_inc(x_185); lean_inc_ref(x_178); -lean_inc(x_183); -lean_inc(x_189); -lean_inc_ref(x_185); +lean_inc(x_180); +lean_inc_ref(x_188); +lean_inc(x_184); +lean_inc(x_177); +lean_inc_ref(x_183); lean_inc_ref(x_19); -x_198 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_checkConstraints(x_19, x_197, x_185, x_188, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); +x_198 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_checkConstraints(x_19, x_197, x_183, x_189, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); if (lean_obj_tag(x_198) == 0) { lean_object* x_199; uint8_t x_200; @@ -33679,18 +33679,18 @@ if (x_200 == 0) lean_object* x_201; lean_dec(x_199); lean_dec(x_197); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); -lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_201 = lean_box(0); @@ -33701,42 +33701,42 @@ goto block_40; else { lean_object* x_202; -lean_inc_ref(x_187); -lean_inc_ref(x_185); +lean_inc_ref(x_179); +lean_inc_ref(x_183); lean_inc_ref(x_19); -x_202 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_collectGuards(x_19, x_185, x_188, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); +x_202 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_collectGuards(x_19, x_183, x_189, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); if (lean_obj_tag(x_202) == 0) { lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; x_203 = lean_ctor_get(x_202, 0); lean_inc(x_203); lean_dec_ref(x_202); -x_204 = l_Lean_mkAppN(x_185, x_188); +x_204 = l_Lean_mkAppN(x_183, x_189); x_205 = lean_unsigned_to_nat(0u); -x_206 = lean_array_get_size(x_188); +x_206 = lean_array_get_size(x_189); x_207 = lean_nat_dec_lt(x_205, x_206); if (x_207 == 0) { uint8_t x_208; lean_object* x_209; x_208 = lean_unbox(x_199); lean_dec(x_199); -x_209 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_208, x_190, x_190, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); -x_143 = x_176; -x_144 = x_177; -x_145 = x_178; -x_146 = x_179; -x_147 = x_181; -x_148 = x_182; -x_149 = x_203; -x_150 = x_204; -x_151 = x_183; -x_152 = x_184; -x_153 = x_205; -x_154 = x_187; -x_155 = x_188; -x_156 = x_197; +x_209 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_208, x_190, x_190, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); +x_143 = x_205; +x_144 = x_176; +x_145 = x_206; +x_146 = x_177; +x_147 = x_204; +x_148 = x_178; +x_149 = x_179; +x_150 = x_203; +x_151 = x_180; +x_152 = x_181; +x_153 = x_182; +x_154 = x_184; +x_155 = x_185; +x_156 = x_188; x_157 = x_189; -x_158 = x_206; +x_158 = x_197; x_159 = x_209; goto block_175; } @@ -33747,23 +33747,23 @@ if (x_207 == 0) uint8_t x_210; lean_object* x_211; x_210 = lean_unbox(x_199); lean_dec(x_199); -x_211 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_210, x_190, x_190, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); -x_143 = x_176; -x_144 = x_177; -x_145 = x_178; -x_146 = x_179; -x_147 = x_181; -x_148 = x_182; -x_149 = x_203; -x_150 = x_204; -x_151 = x_183; -x_152 = x_184; -x_153 = x_205; -x_154 = x_187; -x_155 = x_188; -x_156 = x_197; +x_211 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_210, x_190, x_190, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); +x_143 = x_205; +x_144 = x_176; +x_145 = x_206; +x_146 = x_177; +x_147 = x_204; +x_148 = x_178; +x_149 = x_179; +x_150 = x_203; +x_151 = x_180; +x_152 = x_181; +x_153 = x_182; +x_154 = x_184; +x_155 = x_185; +x_156 = x_188; x_157 = x_189; -x_158 = x_206; +x_158 = x_197; x_159 = x_211; goto block_175; } @@ -33773,7 +33773,7 @@ size_t x_212; size_t x_213; uint8_t x_214; lean_object* x_215; x_212 = 0; x_213 = lean_usize_of_nat(x_206); x_214 = lean_unbox(x_199); -x_215 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__4___redArg(x_214, x_190, x_188, x_212, x_213, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); +x_215 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__4___redArg(x_214, x_190, x_189, x_212, x_213, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); if (lean_obj_tag(x_215) == 0) { lean_object* x_216; uint8_t x_217; uint8_t x_218; lean_object* x_219; @@ -33784,45 +33784,45 @@ x_217 = lean_unbox(x_199); lean_dec(x_199); x_218 = lean_unbox(x_216); lean_dec(x_216); -x_219 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_217, x_190, x_218, x_177, x_182, x_189, x_183, x_178, x_181, x_179, x_184, x_187, x_176); -x_143 = x_176; -x_144 = x_177; -x_145 = x_178; -x_146 = x_179; -x_147 = x_181; -x_148 = x_182; -x_149 = x_203; -x_150 = x_204; -x_151 = x_183; -x_152 = x_184; -x_153 = x_205; -x_154 = x_187; -x_155 = x_188; -x_156 = x_197; +x_219 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_217, x_190, x_218, x_176, x_181, x_177, x_184, x_188, x_180, x_178, x_185, x_179, x_182); +x_143 = x_205; +x_144 = x_176; +x_145 = x_206; +x_146 = x_177; +x_147 = x_204; +x_148 = x_178; +x_149 = x_179; +x_150 = x_203; +x_151 = x_180; +x_152 = x_181; +x_153 = x_182; +x_154 = x_184; +x_155 = x_185; +x_156 = x_188; x_157 = x_189; -x_158 = x_206; +x_158 = x_197; x_159 = x_219; goto block_175; } else { lean_dec(x_199); -x_143 = x_176; -x_144 = x_177; -x_145 = x_178; -x_146 = x_179; -x_147 = x_181; -x_148 = x_182; -x_149 = x_203; -x_150 = x_204; -x_151 = x_183; -x_152 = x_184; -x_153 = x_205; -x_154 = x_187; -x_155 = x_188; -x_156 = x_197; +x_143 = x_205; +x_144 = x_176; +x_145 = x_206; +x_146 = x_177; +x_147 = x_204; +x_148 = x_178; +x_149 = x_179; +x_150 = x_203; +x_151 = x_180; +x_152 = x_181; +x_153 = x_182; +x_154 = x_184; +x_155 = x_185; +x_156 = x_188; x_157 = x_189; -x_158 = x_206; +x_158 = x_197; x_159 = x_215; goto block_175; } @@ -33834,18 +33834,18 @@ else lean_object* x_220; lean_dec(x_199); lean_dec(x_197); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); -lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_220 = lean_ctor_get(x_202, 0); @@ -33861,18 +33861,18 @@ else { lean_object* x_221; lean_dec(x_197); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); -lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_221 = lean_ctor_get(x_198, 0); @@ -33888,18 +33888,18 @@ else lean_object* x_222; lean_dec(x_196); lean_dec(x_194); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); -lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_222 = lean_box(0); @@ -33912,18 +33912,18 @@ else { lean_object* x_223; lean_dec(x_194); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); -lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_223 = lean_ctor_get(x_195, 0); @@ -33938,19 +33938,19 @@ else { lean_object* x_224; lean_dec(x_192); -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); -lean_dec_ref(x_180); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_224 = lean_box(0); @@ -33962,19 +33962,19 @@ goto block_40; else { lean_object* x_225; -lean_dec(x_189); +lean_dec_ref(x_189); lean_dec_ref(x_188); lean_dec_ref(x_187); -lean_dec_ref(x_185); +lean_dec(x_185); lean_dec(x_184); -lean_dec(x_183); +lean_dec_ref(x_183); lean_dec(x_182); lean_dec(x_181); -lean_dec_ref(x_180); +lean_dec(x_180); lean_dec_ref(x_179); lean_dec_ref(x_178); -lean_dec_ref(x_177); -lean_dec(x_176); +lean_dec(x_177); +lean_dec_ref(x_176); lean_dec(x_49); lean_dec_ref(x_19); x_225 = lean_ctor_get(x_191, 0); @@ -34058,20 +34058,20 @@ if (x_255 == 0) if (x_241 == 0) { lean_free_object(x_249); -x_176 = x_236; -x_177 = x_227; -x_178 = x_231; -x_179 = x_233; -x_180 = x_252; -x_181 = x_232; -x_182 = x_228; -x_183 = x_230; -x_184 = x_234; -x_185 = x_239; +x_176 = x_227; +x_177 = x_229; +x_178 = x_233; +x_179 = x_235; +x_180 = x_232; +x_181 = x_228; +x_182 = x_236; +x_183 = x_239; +x_184 = x_230; +x_185 = x_234; x_186 = lean_box(0); -x_187 = x_235; -x_188 = x_250; -x_189 = x_229; +x_187 = x_252; +x_188 = x_231; +x_189 = x_250; x_190 = x_241; goto block_226; } @@ -34187,20 +34187,20 @@ else uint8_t x_266; lean_free_object(x_249); x_266 = 0; -x_176 = x_236; -x_177 = x_227; -x_178 = x_231; -x_179 = x_233; -x_180 = x_252; -x_181 = x_232; -x_182 = x_228; -x_183 = x_230; -x_184 = x_234; -x_185 = x_239; +x_176 = x_227; +x_177 = x_229; +x_178 = x_233; +x_179 = x_235; +x_180 = x_232; +x_181 = x_228; +x_182 = x_236; +x_183 = x_239; +x_184 = x_230; +x_185 = x_234; x_186 = lean_box(0); -x_187 = x_235; -x_188 = x_250; -x_189 = x_229; +x_187 = x_252; +x_188 = x_231; +x_189 = x_250; x_190 = x_266; goto block_226; } @@ -34217,20 +34217,20 @@ if (x_269 == 0) { if (x_241 == 0) { -x_176 = x_236; -x_177 = x_227; -x_178 = x_231; -x_179 = x_233; -x_180 = x_267; -x_181 = x_232; -x_182 = x_228; -x_183 = x_230; -x_184 = x_234; -x_185 = x_239; +x_176 = x_227; +x_177 = x_229; +x_178 = x_233; +x_179 = x_235; +x_180 = x_232; +x_181 = x_228; +x_182 = x_236; +x_183 = x_239; +x_184 = x_230; +x_185 = x_234; x_186 = lean_box(0); -x_187 = x_235; -x_188 = x_250; -x_189 = x_229; +x_187 = x_267; +x_188 = x_231; +x_189 = x_250; x_190 = x_241; goto block_226; } @@ -34342,20 +34342,20 @@ else { uint8_t x_281; x_281 = 0; -x_176 = x_236; -x_177 = x_227; -x_178 = x_231; -x_179 = x_233; -x_180 = x_267; -x_181 = x_232; -x_182 = x_228; -x_183 = x_230; -x_184 = x_234; -x_185 = x_239; +x_176 = x_227; +x_177 = x_229; +x_178 = x_233; +x_179 = x_235; +x_180 = x_232; +x_181 = x_228; +x_182 = x_236; +x_183 = x_239; +x_184 = x_230; +x_185 = x_234; x_186 = lean_box(0); -x_187 = x_235; -x_188 = x_250; -x_189 = x_229; +x_187 = x_267; +x_188 = x_231; +x_189 = x_250; x_190 = x_281; goto block_226; } @@ -34587,7 +34587,7 @@ lean_inc_ref(x_317); x_342 = l_Lean_Meta_Grind_markTheoremInstance___redArg(x_317, x_320, x_4); if (lean_obj_tag(x_342) == 0) { -lean_object* x_343; uint8_t 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_370; uint8_t 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_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_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; uint8_t x_463; 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; uint8_t x_544; +lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; uint8_t 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_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; uint8_t 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_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_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; uint8_t x_463; 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; uint8_t x_544; x_343 = lean_ctor_get(x_342, 0); lean_inc(x_343); lean_dec_ref(x_342); @@ -34719,7 +34719,7 @@ goto block_341; block_369: { lean_object* x_360; lean_object* x_361; uint8_t x_362; uint8_t x_363; uint8_t x_364; lean_object* x_365; -x_360 = l_Lean_instantiateMVars___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__0___redArg(x_348, x_356); +x_360 = l_Lean_instantiateMVars___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__0___redArg(x_344, x_356); x_361 = lean_ctor_get(x_360, 0); lean_inc(x_361); lean_dec_ref(x_360); @@ -34727,16 +34727,16 @@ x_362 = 0; x_363 = lean_unbox(x_343); x_364 = lean_unbox(x_343); lean_dec(x_343); -x_365 = l_Lean_Meta_mkLambdaFVars(x_345, x_361, x_344, x_363, x_344, x_364, x_362, x_355, x_356, x_357, x_358); -lean_dec_ref(x_345); +x_365 = l_Lean_Meta_mkLambdaFVars(x_348, x_361, x_347, x_363, x_347, x_364, x_362, x_355, x_356, x_357, x_358); +lean_dec_ref(x_348); if (lean_obj_tag(x_365) == 0) { lean_object* x_366; lean_object* x_367; x_366 = lean_ctor_get(x_365, 0); lean_inc(x_366); lean_dec_ref(x_365); -x_367 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_315, x_366, x_347, x_346, x_349, x_350, x_351, x_352, x_353, x_354, x_355, x_356, x_357, x_358); -lean_dec(x_347); +x_367 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_315, x_366, x_345, x_346, x_349, x_350, x_351, x_352, x_353, x_354, x_355, x_356, x_357, x_358); +lean_dec(x_345); x_338 = x_367; goto block_341; } @@ -34753,8 +34753,8 @@ lean_dec(x_352); lean_dec(x_351); lean_dec(x_350); lean_dec_ref(x_349); -lean_dec(x_347); lean_dec(x_346); +lean_dec(x_345); lean_dec_ref(x_315); x_368 = lean_ctor_get(x_365, 0); lean_inc(x_368); @@ -34771,11 +34771,11 @@ x_386 = lean_box(0); x_387 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__2___closed__0; x_388 = lean_array_size(x_384); x_389 = 0; -lean_inc(x_370); -lean_inc_ref(x_381); -lean_inc(x_380); +lean_inc(x_379); lean_inc_ref(x_374); -x_390 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__2___redArg(x_387, x_386, x_384, x_388, x_389, x_387, x_374, x_380, x_381, x_370); +lean_inc(x_381); +lean_inc_ref(x_373); +x_390 = l___private_Init_Data_Array_Basic_0__Array_forIn_x27Unsafe_loop___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__2___redArg(x_387, x_386, x_384, x_388, x_389, x_387, x_373, x_381, x_374, x_379); if (lean_obj_tag(x_390) == 0) { lean_object* x_391; lean_object* x_392; lean_object* x_393; @@ -34795,21 +34795,21 @@ if (lean_is_exclusive(x_391)) { if (lean_obj_tag(x_392) == 0) { lean_dec(x_393); -x_344 = x_371; -x_345 = x_384; -x_346 = x_377; -x_347 = x_382; -x_348 = x_378; -x_349 = x_372; -x_350 = x_376; -x_351 = x_383; -x_352 = x_379; -x_353 = x_373; -x_354 = x_375; -x_355 = x_374; -x_356 = x_380; -x_357 = x_381; -x_358 = x_370; +x_344 = x_372; +x_345 = x_383; +x_346 = x_375; +x_347 = x_376; +x_348 = x_384; +x_349 = x_370; +x_350 = x_378; +x_351 = x_371; +x_352 = x_380; +x_353 = x_382; +x_354 = x_377; +x_355 = x_373; +x_356 = x_381; +x_357 = x_374; +x_358 = x_379; x_359 = lean_box(0); goto block_369; } @@ -34825,7 +34825,7 @@ lean_object* x_395; lean_object* x_396; x_395 = lean_ctor_get(x_394, 0); lean_inc(x_395); lean_dec_ref(x_394); -x_396 = l_Lean_Meta_Grind_getConfig___redArg(x_373); +x_396 = l_Lean_Meta_Grind_getConfig___redArg(x_382); if (lean_obj_tag(x_396) == 0) { lean_object* x_397; uint8_t x_398; @@ -34838,60 +34838,60 @@ if (x_398 == 0) { lean_dec(x_395); lean_dec(x_393); -x_344 = x_371; -x_345 = x_384; -x_346 = x_377; -x_347 = x_382; -x_348 = x_378; -x_349 = x_372; -x_350 = x_376; -x_351 = x_383; -x_352 = x_379; -x_353 = x_373; -x_354 = x_375; -x_355 = x_374; -x_356 = x_380; -x_357 = x_381; -x_358 = x_370; +x_344 = x_372; +x_345 = x_383; +x_346 = x_375; +x_347 = x_376; +x_348 = x_384; +x_349 = x_370; +x_350 = x_378; +x_351 = x_371; +x_352 = x_380; +x_353 = x_382; +x_354 = x_377; +x_355 = x_373; +x_356 = x_381; +x_357 = x_374; +x_358 = x_379; x_359 = lean_box(0); goto block_369; } else { lean_object* x_399; lean_object* x_400; uint8_t x_401; -x_399 = lean_ctor_get(x_381, 2); +x_399 = lean_ctor_get(x_374, 2); x_400 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___closed__0; x_401 = l_Lean_Option_get___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance_spec__2(x_399, x_400); if (x_401 == 0) { lean_dec(x_395); lean_dec(x_393); -x_344 = x_371; -x_345 = x_384; -x_346 = x_377; -x_347 = x_382; -x_348 = x_378; -x_349 = x_372; -x_350 = x_376; -x_351 = x_383; -x_352 = x_379; -x_353 = x_373; -x_354 = x_375; -x_355 = x_374; -x_356 = x_380; -x_357 = x_381; -x_358 = x_370; +x_344 = x_372; +x_345 = x_383; +x_346 = x_375; +x_347 = x_376; +x_348 = x_384; +x_349 = x_370; +x_350 = x_378; +x_351 = x_371; +x_352 = x_380; +x_353 = x_382; +x_354 = x_377; +x_355 = x_373; +x_356 = x_381; +x_357 = x_374; +x_358 = x_379; x_359 = lean_box(0); goto block_369; } else { lean_object* x_402; -lean_inc(x_370); -lean_inc_ref(x_381); -lean_inc(x_380); +lean_inc(x_379); lean_inc_ref(x_374); -x_402 = lean_infer_type(x_395, x_374, x_380, x_381, x_370); +lean_inc(x_381); +lean_inc_ref(x_373); +x_402 = lean_infer_type(x_395, x_373, x_381, x_374, x_379); if (lean_obj_tag(x_402) == 0) { 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; @@ -34917,25 +34917,25 @@ x_409 = l_Lean_indentExpr(x_403); x_410 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_410, 0, x_408); lean_ctor_set(x_410, 1, x_409); -x_411 = l_Lean_Meta_Grind_reportIssue(x_410, x_379, x_373, x_375, x_374, x_380, x_381, x_370); +x_411 = l_Lean_Meta_Grind_reportIssue(x_410, x_380, x_382, x_377, x_373, x_381, x_374, x_379); if (lean_obj_tag(x_411) == 0) { lean_dec_ref(x_411); -x_344 = x_371; -x_345 = x_384; -x_346 = x_377; -x_347 = x_382; -x_348 = x_378; -x_349 = x_372; -x_350 = x_376; -x_351 = x_383; -x_352 = x_379; -x_353 = x_373; -x_354 = x_375; -x_355 = x_374; -x_356 = x_380; -x_357 = x_381; -x_358 = x_370; +x_344 = x_372; +x_345 = x_383; +x_346 = x_375; +x_347 = x_376; +x_348 = x_384; +x_349 = x_370; +x_350 = x_378; +x_351 = x_371; +x_352 = x_380; +x_353 = x_382; +x_354 = x_377; +x_355 = x_373; +x_356 = x_381; +x_357 = x_374; +x_358 = x_379; x_359 = lean_box(0); goto block_369; } @@ -34943,18 +34943,18 @@ else { lean_dec_ref(x_384); lean_dec(x_383); -lean_dec(x_382); -lean_dec_ref(x_381); +lean_dec_ref(x_382); +lean_dec(x_381); lean_dec(x_380); lean_dec(x_379); -lean_dec_ref(x_378); +lean_dec(x_378); lean_dec(x_377); -lean_dec(x_376); lean_dec(x_375); lean_dec_ref(x_374); lean_dec_ref(x_373); lean_dec_ref(x_372); -lean_dec(x_370); +lean_dec(x_371); +lean_dec_ref(x_370); lean_dec(x_343); lean_dec_ref(x_315); x_338 = x_411; @@ -34967,18 +34967,18 @@ lean_object* x_412; lean_dec(x_393); lean_dec_ref(x_384); lean_dec(x_383); -lean_dec(x_382); -lean_dec_ref(x_381); +lean_dec_ref(x_382); +lean_dec(x_381); lean_dec(x_380); lean_dec(x_379); -lean_dec_ref(x_378); +lean_dec(x_378); lean_dec(x_377); -lean_dec(x_376); lean_dec(x_375); lean_dec_ref(x_374); lean_dec_ref(x_373); lean_dec_ref(x_372); -lean_dec(x_370); +lean_dec(x_371); +lean_dec_ref(x_370); lean_dec(x_343); lean_dec_ref(x_315); x_412 = lean_ctor_get(x_402, 0); @@ -34998,18 +34998,18 @@ lean_dec(x_395); lean_dec(x_393); lean_dec_ref(x_384); lean_dec(x_383); -lean_dec(x_382); -lean_dec_ref(x_381); +lean_dec_ref(x_382); +lean_dec(x_381); lean_dec(x_380); lean_dec(x_379); -lean_dec_ref(x_378); +lean_dec(x_378); lean_dec(x_377); -lean_dec(x_376); lean_dec(x_375); lean_dec_ref(x_374); lean_dec_ref(x_373); lean_dec_ref(x_372); -lean_dec(x_370); +lean_dec(x_371); +lean_dec_ref(x_370); lean_dec(x_343); lean_dec_ref(x_315); x_413 = lean_ctor_get(x_396, 0); @@ -35024,21 +35024,21 @@ else { lean_dec(x_394); lean_dec(x_393); -x_344 = x_371; -x_345 = x_384; -x_346 = x_377; -x_347 = x_382; -x_348 = x_378; -x_349 = x_372; -x_350 = x_376; -x_351 = x_383; -x_352 = x_379; -x_353 = x_373; -x_354 = x_375; -x_355 = x_374; -x_356 = x_380; -x_357 = x_381; -x_358 = x_370; +x_344 = x_372; +x_345 = x_383; +x_346 = x_375; +x_347 = x_376; +x_348 = x_384; +x_349 = x_370; +x_350 = x_378; +x_351 = x_371; +x_352 = x_380; +x_353 = x_382; +x_354 = x_377; +x_355 = x_373; +x_356 = x_381; +x_357 = x_374; +x_358 = x_379; x_359 = lean_box(0); goto block_369; } @@ -35049,18 +35049,18 @@ else lean_object* x_414; lean_dec_ref(x_384); lean_dec(x_383); -lean_dec(x_382); -lean_dec_ref(x_381); +lean_dec_ref(x_382); +lean_dec(x_381); lean_dec(x_380); lean_dec(x_379); -lean_dec_ref(x_378); +lean_dec(x_378); lean_dec(x_377); -lean_dec(x_376); lean_dec(x_375); lean_dec_ref(x_374); lean_dec_ref(x_373); lean_dec_ref(x_372); -lean_dec(x_370); +lean_dec(x_371); +lean_dec_ref(x_370); lean_dec(x_343); lean_dec_ref(x_315); x_414 = lean_ctor_get(x_390, 0); @@ -35083,29 +35083,29 @@ x_434 = lean_unbox(x_433); if (x_434 == 0) { lean_object* x_435; uint8_t x_436; -x_435 = lean_mk_empty_array_with_capacity(x_426); -x_436 = lean_nat_dec_lt(x_426, x_431); +x_435 = lean_mk_empty_array_with_capacity(x_416); +x_436 = lean_nat_dec_lt(x_416, x_418); if (x_436 == 0) { uint8_t x_437; -lean_dec(x_431); -lean_dec_ref(x_428); +lean_dec_ref(x_430); +lean_dec(x_418); x_437 = lean_unbox(x_433); lean_dec(x_433); -x_370 = x_416; -x_371 = x_437; -x_372 = x_417; -x_373 = x_418; -x_374 = x_419; -x_375 = x_420; -x_376 = x_421; -x_377 = x_422; -x_378 = x_423; -x_379 = x_424; -x_380 = x_425; -x_381 = x_427; +x_370 = x_417; +x_371 = x_419; +x_372 = x_420; +x_373 = x_421; +x_374 = x_422; +x_375 = x_423; +x_376 = x_437; +x_377 = x_424; +x_378 = x_425; +x_379 = x_426; +x_380 = x_427; +x_381 = x_428; x_382 = x_429; -x_383 = x_430; +x_383 = x_431; x_384 = x_435; x_385 = lean_box(0); goto block_415; @@ -35113,28 +35113,28 @@ goto block_415; else { uint8_t x_438; -x_438 = lean_nat_dec_le(x_431, x_431); +x_438 = lean_nat_dec_le(x_418, x_418); if (x_438 == 0) { uint8_t x_439; -lean_dec(x_431); -lean_dec_ref(x_428); +lean_dec_ref(x_430); +lean_dec(x_418); x_439 = lean_unbox(x_433); lean_dec(x_433); -x_370 = x_416; -x_371 = x_439; -x_372 = x_417; -x_373 = x_418; -x_374 = x_419; -x_375 = x_420; -x_376 = x_421; -x_377 = x_422; -x_378 = x_423; -x_379 = x_424; -x_380 = x_425; -x_381 = x_427; +x_370 = x_417; +x_371 = x_419; +x_372 = x_420; +x_373 = x_421; +x_374 = x_422; +x_375 = x_423; +x_376 = x_439; +x_377 = x_424; +x_378 = x_425; +x_379 = x_426; +x_380 = x_427; +x_381 = x_428; x_382 = x_429; -x_383 = x_430; +x_383 = x_431; x_384 = x_435; x_385 = lean_box(0); goto block_415; @@ -35143,10 +35143,10 @@ else { size_t x_440; size_t x_441; lean_object* x_442; x_440 = 0; -x_441 = lean_usize_of_nat(x_431); -lean_dec(x_431); -x_442 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__3___redArg(x_428, x_440, x_441, x_435, x_417, x_421, x_430, x_424, x_418, x_420, x_419, x_425, x_427, x_416); -lean_dec_ref(x_428); +x_441 = lean_usize_of_nat(x_418); +lean_dec(x_418); +x_442 = l___private_Init_Data_Array_Basic_0__Array_foldlMUnsafe_fold___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__3___redArg(x_430, x_440, x_441, x_435, x_417, x_425, x_419, x_427, x_429, x_424, x_421, x_428, x_422, x_426); +lean_dec_ref(x_430); if (lean_obj_tag(x_442) == 0) { lean_object* x_443; uint8_t x_444; @@ -35155,20 +35155,20 @@ lean_inc(x_443); lean_dec_ref(x_442); x_444 = lean_unbox(x_433); lean_dec(x_433); -x_370 = x_416; -x_371 = x_444; -x_372 = x_417; -x_373 = x_418; -x_374 = x_419; -x_375 = x_420; -x_376 = x_421; -x_377 = x_422; -x_378 = x_423; -x_379 = x_424; -x_380 = x_425; -x_381 = x_427; +x_370 = x_417; +x_371 = x_419; +x_372 = x_420; +x_373 = x_421; +x_374 = x_422; +x_375 = x_423; +x_376 = x_444; +x_377 = x_424; +x_378 = x_425; +x_379 = x_426; +x_380 = x_427; +x_381 = x_428; x_382 = x_429; -x_383 = x_430; +x_383 = x_431; x_384 = x_443; x_385 = lean_box(0); goto block_415; @@ -35177,19 +35177,19 @@ else { lean_object* x_445; lean_dec(x_433); -lean_dec(x_430); -lean_dec(x_429); -lean_dec_ref(x_427); +lean_dec(x_431); +lean_dec_ref(x_429); +lean_dec(x_428); +lean_dec(x_427); +lean_dec(x_426); lean_dec(x_425); lean_dec(x_424); -lean_dec_ref(x_423); -lean_dec(x_422); -lean_dec(x_421); -lean_dec(x_420); -lean_dec_ref(x_419); -lean_dec_ref(x_418); +lean_dec(x_423); +lean_dec_ref(x_422); +lean_dec_ref(x_421); +lean_dec_ref(x_420); +lean_dec(x_419); lean_dec_ref(x_417); -lean_dec(x_416); lean_dec(x_343); lean_dec_ref(x_315); x_445 = lean_ctor_get(x_442, 0); @@ -35206,11 +35206,11 @@ else { lean_object* x_446; lean_dec(x_433); -lean_dec(x_431); -lean_dec_ref(x_428); +lean_dec_ref(x_430); +lean_dec(x_418); lean_dec(x_343); -x_446 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_315, x_423, x_429, x_422, x_417, x_421, x_430, x_424, x_418, x_420, x_419, x_425, x_427, x_416); -lean_dec(x_429); +x_446 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance(x_315, x_420, x_431, x_423, x_417, x_425, x_419, x_427, x_429, x_424, x_421, x_428, x_422, x_426); +lean_dec(x_431); x_338 = x_446; goto block_341; } @@ -35219,20 +35219,20 @@ else { lean_object* x_447; lean_dec(x_431); -lean_dec(x_430); -lean_dec(x_429); -lean_dec_ref(x_428); -lean_dec_ref(x_427); +lean_dec_ref(x_430); +lean_dec_ref(x_429); +lean_dec(x_428); +lean_dec(x_427); +lean_dec(x_426); lean_dec(x_425); lean_dec(x_424); -lean_dec_ref(x_423); -lean_dec(x_422); -lean_dec(x_421); -lean_dec(x_420); -lean_dec_ref(x_419); -lean_dec_ref(x_418); +lean_dec(x_423); +lean_dec_ref(x_422); +lean_dec_ref(x_421); +lean_dec_ref(x_420); +lean_dec(x_419); +lean_dec(x_418); lean_dec_ref(x_417); -lean_dec(x_416); lean_dec(x_343); lean_dec_ref(x_315); x_447 = lean_ctor_get(x_432, 0); @@ -35246,17 +35246,17 @@ goto block_327; block_499: { lean_object* x_464; -lean_inc(x_449); -lean_inc_ref(x_460); -lean_inc(x_457); +lean_inc(x_455); lean_inc_ref(x_452); -lean_inc(x_454); +lean_inc(x_458); lean_inc_ref(x_451); -lean_inc(x_456); -lean_inc(x_462); -lean_inc(x_455); -lean_inc_ref(x_450); -x_464 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_applyAssignment(x_461, x_1, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); +lean_inc(x_453); +lean_inc_ref(x_461); +lean_inc(x_457); +lean_inc(x_450); +lean_inc(x_454); +lean_inc_ref(x_449); +x_464 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_applyAssignment(x_462, x_1, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); if (lean_obj_tag(x_464) == 0) { lean_object* x_465; lean_object* x_466; @@ -35270,12 +35270,12 @@ lean_object* x_467; lean_object* x_468; x_467 = lean_ctor_get(x_465, 1); lean_inc(x_467); lean_dec(x_465); -lean_inc(x_449); -lean_inc_ref(x_460); -lean_inc(x_457); +lean_inc(x_455); lean_inc_ref(x_452); -lean_inc_ref(x_450); -x_468 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_synthesizeInsts(x_461, x_453, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); +lean_inc(x_458); +lean_inc_ref(x_451); +lean_inc_ref(x_449); +x_468 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_synthesizeInsts(x_462, x_460, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); if (lean_obj_tag(x_468) == 0) { lean_object* x_469; @@ -35289,17 +35289,17 @@ lean_dec_ref(x_469); x_470 = lean_ctor_get(x_467, 1); lean_inc(x_470); lean_dec(x_467); -lean_inc(x_449); -lean_inc_ref(x_460); -lean_inc(x_457); +lean_inc(x_455); lean_inc_ref(x_452); -lean_inc(x_454); +lean_inc(x_458); lean_inc_ref(x_451); -lean_inc(x_456); -lean_inc(x_462); -lean_inc_ref(x_458); +lean_inc(x_453); +lean_inc_ref(x_461); +lean_inc(x_457); +lean_inc(x_450); +lean_inc_ref(x_456); lean_inc_ref(x_315); -x_471 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_checkConstraints(x_315, x_470, x_458, x_461, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); +x_471 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_checkConstraints(x_315, x_470, x_456, x_462, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); if (lean_obj_tag(x_471) == 0) { lean_object* x_472; uint8_t x_473; @@ -35312,18 +35312,18 @@ if (x_473 == 0) lean_object* x_474; lean_dec(x_472); lean_dec(x_470); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); -lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_474 = lean_box(0); @@ -35334,42 +35334,42 @@ goto block_334; else { lean_object* x_475; -lean_inc_ref(x_460); -lean_inc_ref(x_458); +lean_inc_ref(x_452); +lean_inc_ref(x_456); lean_inc_ref(x_315); -x_475 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_collectGuards(x_315, x_458, x_461, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); +x_475 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_collectGuards(x_315, x_456, x_462, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); if (lean_obj_tag(x_475) == 0) { lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; uint8_t x_480; x_476 = lean_ctor_get(x_475, 0); lean_inc(x_476); lean_dec_ref(x_475); -x_477 = l_Lean_mkAppN(x_458, x_461); +x_477 = l_Lean_mkAppN(x_456, x_462); x_478 = lean_unsigned_to_nat(0u); -x_479 = lean_array_get_size(x_461); +x_479 = lean_array_get_size(x_462); x_480 = lean_nat_dec_lt(x_478, x_479); if (x_480 == 0) { uint8_t x_481; lean_object* x_482; x_481 = lean_unbox(x_472); lean_dec(x_472); -x_482 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_481, x_463, x_463, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); -x_416 = x_449; -x_417 = x_450; -x_418 = x_451; -x_419 = x_452; -x_420 = x_454; -x_421 = x_455; -x_422 = x_476; -x_423 = x_477; -x_424 = x_456; -x_425 = x_457; -x_426 = x_478; -x_427 = x_460; -x_428 = x_461; -x_429 = x_470; +x_482 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_481, x_463, x_463, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); +x_416 = x_478; +x_417 = x_449; +x_418 = x_479; +x_419 = x_450; +x_420 = x_477; +x_421 = x_451; +x_422 = x_452; +x_423 = x_476; +x_424 = x_453; +x_425 = x_454; +x_426 = x_455; +x_427 = x_457; +x_428 = x_458; +x_429 = x_461; x_430 = x_462; -x_431 = x_479; +x_431 = x_470; x_432 = x_482; goto block_448; } @@ -35380,23 +35380,23 @@ if (x_480 == 0) uint8_t x_483; lean_object* x_484; x_483 = lean_unbox(x_472); lean_dec(x_472); -x_484 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_483, x_463, x_463, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); -x_416 = x_449; -x_417 = x_450; -x_418 = x_451; -x_419 = x_452; -x_420 = x_454; -x_421 = x_455; -x_422 = x_476; -x_423 = x_477; -x_424 = x_456; -x_425 = x_457; -x_426 = x_478; -x_427 = x_460; -x_428 = x_461; -x_429 = x_470; +x_484 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_483, x_463, x_463, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); +x_416 = x_478; +x_417 = x_449; +x_418 = x_479; +x_419 = x_450; +x_420 = x_477; +x_421 = x_451; +x_422 = x_452; +x_423 = x_476; +x_424 = x_453; +x_425 = x_454; +x_426 = x_455; +x_427 = x_457; +x_428 = x_458; +x_429 = x_461; x_430 = x_462; -x_431 = x_479; +x_431 = x_470; x_432 = x_484; goto block_448; } @@ -35406,7 +35406,7 @@ size_t x_485; size_t x_486; uint8_t x_487; lean_object* x_488; x_485 = 0; x_486 = lean_usize_of_nat(x_479); x_487 = lean_unbox(x_472); -x_488 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__4___redArg(x_487, x_463, x_461, x_485, x_486, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); +x_488 = l___private_Init_Data_Array_Basic_0__Array_anyMUnsafe_any___at___00__private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem_spec__4___redArg(x_487, x_463, x_462, x_485, x_486, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); if (lean_obj_tag(x_488) == 0) { lean_object* x_489; uint8_t x_490; uint8_t x_491; lean_object* x_492; @@ -35417,45 +35417,45 @@ x_490 = lean_unbox(x_472); lean_dec(x_472); x_491 = lean_unbox(x_489); lean_dec(x_489); -x_492 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_490, x_463, x_491, x_450, x_455, x_462, x_456, x_451, x_454, x_452, x_457, x_460, x_449); -x_416 = x_449; -x_417 = x_450; -x_418 = x_451; -x_419 = x_452; -x_420 = x_454; -x_421 = x_455; -x_422 = x_476; -x_423 = x_477; -x_424 = x_456; -x_425 = x_457; -x_426 = x_478; -x_427 = x_460; -x_428 = x_461; -x_429 = x_470; +x_492 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lam__1(x_490, x_463, x_491, x_449, x_454, x_450, x_457, x_461, x_453, x_451, x_458, x_452, x_455); +x_416 = x_478; +x_417 = x_449; +x_418 = x_479; +x_419 = x_450; +x_420 = x_477; +x_421 = x_451; +x_422 = x_452; +x_423 = x_476; +x_424 = x_453; +x_425 = x_454; +x_426 = x_455; +x_427 = x_457; +x_428 = x_458; +x_429 = x_461; x_430 = x_462; -x_431 = x_479; +x_431 = x_470; x_432 = x_492; goto block_448; } else { lean_dec(x_472); -x_416 = x_449; -x_417 = x_450; -x_418 = x_451; -x_419 = x_452; -x_420 = x_454; -x_421 = x_455; -x_422 = x_476; -x_423 = x_477; -x_424 = x_456; -x_425 = x_457; -x_426 = x_478; -x_427 = x_460; -x_428 = x_461; -x_429 = x_470; +x_416 = x_478; +x_417 = x_449; +x_418 = x_479; +x_419 = x_450; +x_420 = x_477; +x_421 = x_451; +x_422 = x_452; +x_423 = x_476; +x_424 = x_453; +x_425 = x_454; +x_426 = x_455; +x_427 = x_457; +x_428 = x_458; +x_429 = x_461; x_430 = x_462; -x_431 = x_479; +x_431 = x_470; x_432 = x_488; goto block_448; } @@ -35467,18 +35467,18 @@ else lean_object* x_493; lean_dec(x_472); lean_dec(x_470); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); -lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_493 = lean_ctor_get(x_475, 0); @@ -35494,18 +35494,18 @@ else { lean_object* x_494; lean_dec(x_470); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); -lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_494 = lean_ctor_get(x_471, 0); @@ -35521,18 +35521,18 @@ else lean_object* x_495; lean_dec(x_469); lean_dec(x_467); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); -lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_495 = lean_box(0); @@ -35545,18 +35545,18 @@ else { lean_object* x_496; lean_dec(x_467); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); -lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_496 = lean_ctor_get(x_468, 0); @@ -35571,19 +35571,19 @@ else { lean_object* x_497; lean_dec(x_465); -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); -lean_dec_ref(x_453); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_497 = lean_box(0); @@ -35595,19 +35595,19 @@ goto block_334; else { lean_object* x_498; -lean_dec(x_462); +lean_dec_ref(x_462); lean_dec_ref(x_461); lean_dec_ref(x_460); -lean_dec_ref(x_458); +lean_dec(x_458); lean_dec(x_457); -lean_dec(x_456); +lean_dec_ref(x_456); lean_dec(x_455); lean_dec(x_454); -lean_dec_ref(x_453); +lean_dec(x_453); lean_dec_ref(x_452); lean_dec_ref(x_451); -lean_dec_ref(x_450); -lean_dec(x_449); +lean_dec(x_450); +lean_dec_ref(x_449); lean_dec(x_343); lean_dec_ref(x_315); x_498 = lean_ctor_get(x_464, 0); @@ -35694,20 +35694,20 @@ if (x_527 == 0) if (x_514 == 0) { lean_dec(x_525); -x_449 = x_509; -x_450 = x_500; -x_451 = x_504; -x_452 = x_506; -x_453 = x_524; -x_454 = x_505; -x_455 = x_501; -x_456 = x_503; -x_457 = x_507; -x_458 = x_512; +x_449 = x_500; +x_450 = x_502; +x_451 = x_506; +x_452 = x_508; +x_453 = x_505; +x_454 = x_501; +x_455 = x_509; +x_456 = x_512; +x_457 = x_503; +x_458 = x_507; x_459 = lean_box(0); -x_460 = x_508; -x_461 = x_523; -x_462 = x_502; +x_460 = x_524; +x_461 = x_504; +x_462 = x_523; x_463 = x_514; goto block_499; } @@ -35828,20 +35828,20 @@ else uint8_t x_539; lean_dec(x_525); x_539 = 0; -x_449 = x_509; -x_450 = x_500; -x_451 = x_504; -x_452 = x_506; -x_453 = x_524; -x_454 = x_505; -x_455 = x_501; -x_456 = x_503; -x_457 = x_507; -x_458 = x_512; +x_449 = x_500; +x_450 = x_502; +x_451 = x_506; +x_452 = x_508; +x_453 = x_505; +x_454 = x_501; +x_455 = x_509; +x_456 = x_512; +x_457 = x_503; +x_458 = x_507; x_459 = lean_box(0); -x_460 = x_508; -x_461 = x_523; -x_462 = x_502; +x_460 = x_524; +x_461 = x_504; +x_462 = x_523; x_463 = x_539; goto block_499; } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/MatchCond.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/MatchCond.c index 2ed7816cc72e..2b4232e8f625 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/MatchCond.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/MatchCond.c @@ -4938,7 +4938,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_MatchCond_0__Lean_Meta_Grind_mkMatchCondProof_x3f_go_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; uint8_t 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_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; uint8_t x_287; 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_553; lean_object* x_554; +lean_object* x_12; uint8_t x_16; uint8_t 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; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; 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; uint8_t x_287; 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_553; lean_object* x_554; x_553 = l___private_Init_While_0__Lean_Loop_forIn_loop___at___00__private_Init_While_0__Lean_Loop_forIn_loop___at___00__private_Lean_Meta_Tactic_Grind_MatchCond_0__Lean_Meta_Grind_isSatisfied_spec__2_spec__3___closed__3; x_554 = l_Lean_isTracingEnabledFor___at___00__private_Lean_Meta_Tactic_Grind_MatchCond_0__Lean_Meta_Grind_isSatisfied_spec__0___redArg(x_553, x_9); if (lean_obj_tag(x_554) == 0) @@ -5140,7 +5140,7 @@ lean_dec(x_24); lean_dec(x_23); lean_dec_ref(x_20); lean_dec_ref(x_1); -if (x_21 == 0) +if (x_17 == 0) { lean_object* x_32; lean_object* x_33; lean_dec(x_30); @@ -5148,8 +5148,8 @@ lean_dec_ref(x_29); lean_dec(x_28); lean_dec_ref(x_27); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_18); -lean_dec_ref(x_17); x_32 = lean_box(0); x_33 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_33, 0, x_32); @@ -5174,8 +5174,8 @@ lean_inc(x_30); lean_inc_ref(x_29); lean_inc(x_28); lean_inc_ref(x_27); -lean_inc_ref(x_17); -x_36 = l_Lean_Meta_normLitValue(x_17, x_27, x_28, x_29, x_30); +lean_inc_ref(x_21); +x_36 = l_Lean_Meta_normLitValue(x_21, x_27, x_28, x_29, x_30); if (lean_obj_tag(x_36) == 0) { uint8_t x_37; @@ -5195,7 +5195,7 @@ lean_inc(x_30); lean_inc_ref(x_29); lean_inc(x_28); lean_inc_ref(x_27); -x_40 = l_Lean_Meta_mkEq(x_18, x_17, x_27, x_28, x_29, x_30); +x_40 = l_Lean_Meta_mkEq(x_18, x_21, x_27, x_28, x_29, x_30); if (lean_obj_tag(x_40) == 0) { lean_object* x_41; lean_object* x_42; lean_object* x_43; @@ -5286,8 +5286,8 @@ lean_dec_ref(x_29); lean_dec(x_28); lean_dec_ref(x_27); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_18); -lean_dec_ref(x_17); x_58 = lean_box(0); lean_ctor_set(x_36, 0, x_58); return x_36; @@ -5309,7 +5309,7 @@ lean_inc(x_30); lean_inc_ref(x_29); lean_inc(x_28); lean_inc_ref(x_27); -x_61 = l_Lean_Meta_mkEq(x_18, x_17, x_27, x_28, x_29, x_30); +x_61 = l_Lean_Meta_mkEq(x_18, x_21, x_27, x_28, x_29, x_30); if (lean_obj_tag(x_61) == 0) { lean_object* x_62; lean_object* x_63; lean_object* x_64; @@ -5397,8 +5397,8 @@ lean_dec_ref(x_29); lean_dec(x_28); lean_dec_ref(x_27); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_18); -lean_dec_ref(x_17); x_76 = lean_box(0); x_77 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_77, 0, x_76); @@ -5415,8 +5415,8 @@ lean_dec_ref(x_29); lean_dec(x_28); lean_dec_ref(x_27); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_18); -lean_dec_ref(x_17); x_78 = !lean_is_exclusive(x_36); if (x_78 == 0) { @@ -5442,8 +5442,8 @@ lean_dec_ref(x_29); lean_dec(x_28); lean_dec_ref(x_27); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_18); -lean_dec_ref(x_17); x_81 = !lean_is_exclusive(x_34); if (x_81 == 0) { @@ -5489,7 +5489,7 @@ lean_inc(x_30); lean_inc_ref(x_29); lean_inc(x_28); lean_inc_ref(x_27); -x_88 = l_Lean_Meta_isConstructorApp_x3f(x_17, x_27, x_28, x_29, x_30); +x_88 = l_Lean_Meta_isConstructorApp_x3f(x_21, x_27, x_28, x_29, x_30); if (lean_obj_tag(x_88) == 0) { uint8_t x_89; @@ -6483,8 +6483,8 @@ lean_dec_ref(x_25); lean_dec(x_24); lean_dec(x_23); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_20); -lean_dec_ref(x_17); lean_dec_ref(x_1); x_224 = lean_box(0); lean_ctor_set(x_84, 0, x_224); @@ -6507,7 +6507,7 @@ lean_inc(x_30); lean_inc_ref(x_29); lean_inc(x_28); lean_inc_ref(x_27); -x_227 = l_Lean_Meta_isConstructorApp_x3f(x_17, x_27, x_28, x_29, x_30); +x_227 = l_Lean_Meta_isConstructorApp_x3f(x_21, x_27, x_28, x_29, x_30); if (lean_obj_tag(x_227) == 0) { lean_object* x_228; lean_object* x_229; @@ -6833,8 +6833,8 @@ lean_dec_ref(x_25); lean_dec(x_24); lean_dec(x_23); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_20); -lean_dec_ref(x_17); lean_dec_ref(x_1); x_268 = lean_box(0); x_269 = lean_alloc_ctor(0, 1, 0); @@ -6855,8 +6855,8 @@ lean_dec_ref(x_25); lean_dec(x_24); lean_dec(x_23); lean_dec_ref(x_22); +lean_dec_ref(x_21); lean_dec_ref(x_20); -lean_dec_ref(x_17); lean_dec_ref(x_1); x_270 = !lean_is_exclusive(x_84); if (x_270 == 0) @@ -6879,18 +6879,18 @@ return x_272; block_359: { lean_object* x_288; uint8_t x_289; uint8_t x_290; lean_object* x_291; -x_288 = lean_ctor_get(x_279, 0); +x_288 = lean_ctor_get(x_278, 0); lean_inc_ref(x_288); -x_289 = lean_ctor_get_uint8(x_279, sizeof(void*)*11 + 1); -x_290 = lean_ctor_get_uint8(x_279, sizeof(void*)*11 + 2); -lean_dec_ref(x_279); -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +x_289 = lean_ctor_get_uint8(x_278, sizeof(void*)*11 + 1); +x_290 = lean_ctor_get_uint8(x_278, sizeof(void*)*11 + 2); +lean_dec_ref(x_278); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -lean_inc_ref(x_281); +lean_inc_ref(x_286); lean_inc_ref(x_288); -x_291 = l_Lean_Meta_Grind_hasSameType(x_288, x_281, x_276, x_277, x_282, x_284); +x_291 = l_Lean_Meta_Grind_hasSameType(x_288, x_286, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_291) == 0) { uint8_t x_292; @@ -6906,16 +6906,16 @@ lean_object* x_295; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); -lean_dec_ref(x_274); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_295 = lean_box(0); @@ -6928,27 +6928,27 @@ lean_free_object(x_291); if (x_287 == 0) { lean_object* x_296; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -lean_inc(x_278); -lean_inc_ref(x_283); -lean_inc(x_280); -lean_inc(x_275); +lean_inc(x_281); +lean_inc_ref(x_284); +lean_inc(x_283); +lean_inc(x_277); lean_inc_ref(x_288); -x_296 = lean_grind_mk_eq_proof(x_288, x_274, x_275, x_280, x_283, x_278, x_276, x_277, x_282, x_284); +x_296 = lean_grind_mk_eq_proof(x_288, x_282, x_277, x_283, x_284, x_281, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_296) == 0) { lean_object* x_297; lean_object* x_298; x_297 = lean_ctor_get(x_296, 0); lean_inc(x_297); lean_dec_ref(x_296); -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_298 = l_Lean_Meta_mkEqTrans(x_297, x_2, x_276, x_277, x_282, x_284); +x_298 = l_Lean_Meta_mkEqTrans(x_297, x_2, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_298) == 0) { lean_object* x_299; uint8_t x_300; @@ -6958,20 +6958,20 @@ lean_dec_ref(x_298); x_300 = lean_unbox(x_293); lean_dec(x_293); x_16 = x_300; -x_17 = x_281; +x_17 = x_289; x_18 = x_288; x_19 = x_290; -x_20 = x_286; -x_21 = x_289; +x_20 = x_279; +x_21 = x_286; x_22 = x_299; -x_23 = x_275; -x_24 = x_280; -x_25 = x_283; -x_26 = x_278; +x_23 = x_277; +x_24 = x_283; +x_25 = x_284; +x_26 = x_281; x_27 = x_276; -x_28 = x_277; -x_29 = x_282; -x_30 = x_284; +x_28 = x_274; +x_29 = x_280; +x_30 = x_285; x_31 = lean_box(0); goto block_273; } @@ -6981,15 +6981,15 @@ uint8_t x_301; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_301 = !lean_is_exclusive(x_298); if (x_301 == 0) @@ -7014,15 +7014,15 @@ uint8_t x_304; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_304 = !lean_is_exclusive(x_296); @@ -7045,27 +7045,27 @@ return x_306; else { lean_object* x_307; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -lean_inc(x_278); -lean_inc_ref(x_283); -lean_inc(x_280); -lean_inc(x_275); +lean_inc(x_281); +lean_inc_ref(x_284); +lean_inc(x_283); +lean_inc(x_277); lean_inc_ref(x_288); -x_307 = lean_grind_mk_heq_proof(x_288, x_274, x_275, x_280, x_283, x_278, x_276, x_277, x_282, x_284); +x_307 = lean_grind_mk_heq_proof(x_288, x_282, x_277, x_283, x_284, x_281, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_307) == 0) { lean_object* x_308; lean_object* x_309; x_308 = lean_ctor_get(x_307, 0); lean_inc(x_308); lean_dec_ref(x_307); -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_309 = l_Lean_Meta_mkHEqTrans(x_308, x_2, x_276, x_277, x_282, x_284); +x_309 = l_Lean_Meta_mkHEqTrans(x_308, x_2, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_309) == 0) { lean_object* x_310; uint8_t x_311; lean_object* x_312; @@ -7073,11 +7073,11 @@ x_310 = lean_ctor_get(x_309, 0); lean_inc(x_310); lean_dec_ref(x_309); x_311 = 0; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_312 = l_Lean_Meta_mkEqOfHEq(x_310, x_311, x_276, x_277, x_282, x_284); +x_312 = l_Lean_Meta_mkEqOfHEq(x_310, x_311, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_312) == 0) { lean_object* x_313; uint8_t x_314; @@ -7087,20 +7087,20 @@ lean_dec_ref(x_312); x_314 = lean_unbox(x_293); lean_dec(x_293); x_16 = x_314; -x_17 = x_281; +x_17 = x_289; x_18 = x_288; x_19 = x_290; -x_20 = x_286; -x_21 = x_289; +x_20 = x_279; +x_21 = x_286; x_22 = x_313; -x_23 = x_275; -x_24 = x_280; -x_25 = x_283; -x_26 = x_278; +x_23 = x_277; +x_24 = x_283; +x_25 = x_284; +x_26 = x_281; x_27 = x_276; -x_28 = x_277; -x_29 = x_282; -x_30 = x_284; +x_28 = x_274; +x_29 = x_280; +x_30 = x_285; x_31 = lean_box(0); goto block_273; } @@ -7110,15 +7110,15 @@ uint8_t x_315; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_315 = !lean_is_exclusive(x_312); if (x_315 == 0) @@ -7143,15 +7143,15 @@ uint8_t x_318; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_318 = !lean_is_exclusive(x_309); if (x_318 == 0) @@ -7176,15 +7176,15 @@ uint8_t x_321; lean_dec(x_293); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_321 = !lean_is_exclusive(x_307); @@ -7219,16 +7219,16 @@ lean_object* x_326; lean_object* x_327; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); -lean_dec_ref(x_274); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_326 = lean_box(0); @@ -7241,27 +7241,27 @@ else if (x_287 == 0) { lean_object* x_328; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -lean_inc(x_278); -lean_inc_ref(x_283); -lean_inc(x_280); -lean_inc(x_275); +lean_inc(x_281); +lean_inc_ref(x_284); +lean_inc(x_283); +lean_inc(x_277); lean_inc_ref(x_288); -x_328 = lean_grind_mk_eq_proof(x_288, x_274, x_275, x_280, x_283, x_278, x_276, x_277, x_282, x_284); +x_328 = lean_grind_mk_eq_proof(x_288, x_282, x_277, x_283, x_284, x_281, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_328) == 0) { lean_object* x_329; lean_object* x_330; x_329 = lean_ctor_get(x_328, 0); lean_inc(x_329); lean_dec_ref(x_328); -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_330 = l_Lean_Meta_mkEqTrans(x_329, x_2, x_276, x_277, x_282, x_284); +x_330 = l_Lean_Meta_mkEqTrans(x_329, x_2, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_330) == 0) { lean_object* x_331; uint8_t x_332; @@ -7271,20 +7271,20 @@ lean_dec_ref(x_330); x_332 = lean_unbox(x_324); lean_dec(x_324); x_16 = x_332; -x_17 = x_281; +x_17 = x_289; x_18 = x_288; x_19 = x_290; -x_20 = x_286; -x_21 = x_289; +x_20 = x_279; +x_21 = x_286; x_22 = x_331; -x_23 = x_275; -x_24 = x_280; -x_25 = x_283; -x_26 = x_278; +x_23 = x_277; +x_24 = x_283; +x_25 = x_284; +x_26 = x_281; x_27 = x_276; -x_28 = x_277; -x_29 = x_282; -x_30 = x_284; +x_28 = x_274; +x_29 = x_280; +x_30 = x_285; x_31 = lean_box(0); goto block_273; } @@ -7294,15 +7294,15 @@ lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_333 = lean_ctor_get(x_330, 0); lean_inc(x_333); @@ -7328,15 +7328,15 @@ lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_336 = lean_ctor_get(x_328, 0); @@ -7360,27 +7360,27 @@ return x_338; else { lean_object* x_339; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -lean_inc(x_278); -lean_inc_ref(x_283); -lean_inc(x_280); -lean_inc(x_275); +lean_inc(x_281); +lean_inc_ref(x_284); +lean_inc(x_283); +lean_inc(x_277); lean_inc_ref(x_288); -x_339 = lean_grind_mk_heq_proof(x_288, x_274, x_275, x_280, x_283, x_278, x_276, x_277, x_282, x_284); +x_339 = lean_grind_mk_heq_proof(x_288, x_282, x_277, x_283, x_284, x_281, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_339) == 0) { lean_object* x_340; lean_object* x_341; x_340 = lean_ctor_get(x_339, 0); lean_inc(x_340); lean_dec_ref(x_339); -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_341 = l_Lean_Meta_mkHEqTrans(x_340, x_2, x_276, x_277, x_282, x_284); +x_341 = l_Lean_Meta_mkHEqTrans(x_340, x_2, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_341) == 0) { lean_object* x_342; uint8_t x_343; lean_object* x_344; @@ -7388,11 +7388,11 @@ x_342 = lean_ctor_get(x_341, 0); lean_inc(x_342); lean_dec_ref(x_341); x_343 = 0; -lean_inc(x_284); -lean_inc_ref(x_282); -lean_inc(x_277); +lean_inc(x_285); +lean_inc_ref(x_280); +lean_inc(x_274); lean_inc_ref(x_276); -x_344 = l_Lean_Meta_mkEqOfHEq(x_342, x_343, x_276, x_277, x_282, x_284); +x_344 = l_Lean_Meta_mkEqOfHEq(x_342, x_343, x_276, x_274, x_280, x_285); if (lean_obj_tag(x_344) == 0) { lean_object* x_345; uint8_t x_346; @@ -7402,20 +7402,20 @@ lean_dec_ref(x_344); x_346 = lean_unbox(x_324); lean_dec(x_324); x_16 = x_346; -x_17 = x_281; +x_17 = x_289; x_18 = x_288; x_19 = x_290; -x_20 = x_286; -x_21 = x_289; +x_20 = x_279; +x_21 = x_286; x_22 = x_345; -x_23 = x_275; -x_24 = x_280; -x_25 = x_283; -x_26 = x_278; +x_23 = x_277; +x_24 = x_283; +x_25 = x_284; +x_26 = x_281; x_27 = x_276; -x_28 = x_277; -x_29 = x_282; -x_30 = x_284; +x_28 = x_274; +x_29 = x_280; +x_30 = x_285; x_31 = lean_box(0); goto block_273; } @@ -7425,15 +7425,15 @@ lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_347 = lean_ctor_get(x_344, 0); lean_inc(x_347); @@ -7459,15 +7459,15 @@ lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_1); x_350 = lean_ctor_get(x_341, 0); lean_inc(x_350); @@ -7493,15 +7493,15 @@ lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_dec(x_324); lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); -lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_353 = lean_ctor_get(x_339, 0); @@ -7530,16 +7530,16 @@ else uint8_t x_356; lean_dec_ref(x_288); lean_dec_ref(x_286); -lean_dec(x_284); -lean_dec_ref(x_283); +lean_dec(x_285); +lean_dec_ref(x_284); +lean_dec(x_283); lean_dec_ref(x_282); -lean_dec_ref(x_281); -lean_dec(x_280); -lean_dec(x_278); +lean_dec(x_281); +lean_dec_ref(x_280); +lean_dec_ref(x_279); lean_dec(x_277); lean_dec_ref(x_276); -lean_dec(x_275); -lean_dec_ref(x_274); +lean_dec(x_274); lean_dec_ref(x_2); lean_dec_ref(x_1); x_356 = !lean_is_exclusive(x_291); @@ -7632,19 +7632,19 @@ x_388 = lean_ctor_get(x_387, 0); lean_inc(x_388); lean_dec_ref(x_387); x_389 = 0; -x_274 = x_385; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_388; -x_280 = x_361; -x_281 = x_379; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_383; +x_277 = x_360; +x_278 = x_388; +x_279 = x_383; +x_280 = x_366; +x_281 = x_363; +x_282 = x_385; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_379; x_287 = x_389; goto block_359; } @@ -7656,19 +7656,19 @@ x_390 = lean_ctor_get(x_387, 0); lean_inc(x_390); lean_dec_ref(x_387); x_391 = 1; -x_274 = x_385; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_390; -x_280 = x_361; -x_281 = x_379; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_383; +x_277 = x_360; +x_278 = x_390; +x_279 = x_383; +x_280 = x_366; +x_281 = x_363; +x_282 = x_385; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_379; x_287 = x_391; goto block_359; } @@ -7940,19 +7940,19 @@ x_427 = lean_ctor_get(x_426, 0); lean_inc(x_427); lean_dec_ref(x_426); x_428 = 0; -x_274 = x_424; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_427; -x_280 = x_361; -x_281 = x_418; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_422; +x_277 = x_360; +x_278 = x_427; +x_279 = x_422; +x_280 = x_366; +x_281 = x_363; +x_282 = x_424; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_418; x_287 = x_428; goto block_359; } @@ -7964,19 +7964,19 @@ x_429 = lean_ctor_get(x_426, 0); lean_inc(x_429); lean_dec_ref(x_426); x_430 = 1; -x_274 = x_424; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_429; -x_280 = x_361; -x_281 = x_418; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_422; +x_277 = x_360; +x_278 = x_429; +x_279 = x_422; +x_280 = x_366; +x_281 = x_363; +x_282 = x_424; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_418; x_287 = x_430; goto block_359; } @@ -8260,19 +8260,19 @@ x_469 = lean_ctor_get(x_468, 0); lean_inc(x_469); lean_dec_ref(x_468); x_470 = 0; -x_274 = x_466; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_469; -x_280 = x_361; -x_281 = x_459; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_464; +x_277 = x_360; +x_278 = x_469; +x_279 = x_464; +x_280 = x_366; +x_281 = x_363; +x_282 = x_466; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_459; x_287 = x_470; goto block_359; } @@ -8284,19 +8284,19 @@ x_471 = lean_ctor_get(x_468, 0); lean_inc(x_471); lean_dec_ref(x_468); x_472 = 1; -x_274 = x_466; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_471; -x_280 = x_361; -x_281 = x_459; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_464; +x_277 = x_360; +x_278 = x_471; +x_279 = x_464; +x_280 = x_366; +x_281 = x_363; +x_282 = x_466; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_459; x_287 = x_472; goto block_359; } @@ -8622,19 +8622,19 @@ x_517 = lean_ctor_get(x_516, 0); lean_inc(x_517); lean_dec_ref(x_516); x_518 = 0; -x_274 = x_514; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_517; -x_280 = x_361; -x_281 = x_507; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_512; +x_277 = x_360; +x_278 = x_517; +x_279 = x_512; +x_280 = x_366; +x_281 = x_363; +x_282 = x_514; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_507; x_287 = x_518; goto block_359; } @@ -8646,19 +8646,19 @@ x_519 = lean_ctor_get(x_516, 0); lean_inc(x_519); lean_dec_ref(x_516); x_520 = 1; -x_274 = x_514; -x_275 = x_360; +x_274 = x_365; +x_275 = lean_box(0); x_276 = x_364; -x_277 = x_365; -x_278 = x_363; -x_279 = x_519; -x_280 = x_361; -x_281 = x_507; -x_282 = x_366; -x_283 = x_362; -x_284 = x_367; -x_285 = lean_box(0); -x_286 = x_512; +x_277 = x_360; +x_278 = x_519; +x_279 = x_512; +x_280 = x_366; +x_281 = x_363; +x_282 = x_514; +x_283 = x_361; +x_284 = x_362; +x_285 = x_367; +x_286 = x_507; x_287 = x_520; goto block_359; } diff --git a/stage0/stdlib/Lean/Server/Completion/CompletionItemCompression.c b/stage0/stdlib/Lean/Server/Completion/CompletionItemCompression.c index f1a291637722..5f785215b6fe 100644 --- a/stage0/stdlib/Lean/Server/Completion/CompletionItemCompression.c +++ b/stage0/stdlib/Lean/Server/Completion/CompletionItemCompression.c @@ -939,7 +939,7 @@ return x_7; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemFast(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_7; 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_32; lean_object* x_36; lean_object* x_40; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_94; lean_object* x_119; lean_object* x_136; lean_object* x_205; lean_object* x_216; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_241; lean_object* x_250; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; uint8_t x_271; +lean_object* x_3; lean_object* x_7; 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_32; lean_object* x_36; lean_object* x_40; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_94; lean_object* x_119; lean_object* x_136; lean_object* x_205; lean_object* x_216; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_241; lean_object* x_250; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; uint8_t x_271; x_11 = lean_ctor_get(x_2, 0); lean_inc_ref(x_11); x_12 = lean_ctor_get(x_2, 1); @@ -1082,14 +1082,14 @@ goto block_35; } block_74: { -if (lean_obj_tag(x_44) == 1) +if (lean_obj_tag(x_45) == 1) { lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_44, 0); +x_48 = lean_ctor_get(x_45, 0); lean_inc(x_48); -lean_dec_ref(x_44); -x_49 = lean_string_append(x_47, x_45); lean_dec_ref(x_45); +x_49 = lean_string_append(x_47, x_46); +lean_dec_ref(x_46); if (lean_obj_tag(x_48) == 0) { lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; @@ -1098,7 +1098,7 @@ lean_inc(x_50); lean_dec_ref(x_48); x_51 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemDataFast___closed__3; x_52 = lean_string_append(x_49, x_51); -x_53 = l_Lean_Name_toString(x_50, x_46); +x_53 = l_Lean_Name_toString(x_50, x_44); x_54 = l___private_Lean_Data_Json_Printer_0__Lean_Json_needEscape(x_53); if (x_54 == 0) { @@ -1136,7 +1136,7 @@ lean_inc(x_62); lean_dec_ref(x_48); x_63 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemDataFast___closed__4; x_64 = lean_string_append(x_49, x_63); -x_65 = l_Lean_Name_toString(x_62, x_46); +x_65 = l_Lean_Name_toString(x_62, x_44); x_66 = l___private_Lean_Data_Json_Printer_0__Lean_Json_needEscape(x_65); if (x_66 == 0) { @@ -1169,8 +1169,8 @@ goto block_43; } else { -lean_dec_ref(x_45); -lean_dec(x_44); +lean_dec_ref(x_46); +lean_dec(x_45); x_32 = x_47; goto block_35; } @@ -1178,11 +1178,11 @@ goto block_35; block_93: { 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_80 = lean_ctor_get(x_77, 0); +x_80 = lean_ctor_get(x_75, 0); lean_inc(x_80); -x_81 = lean_ctor_get(x_77, 1); +x_81 = lean_ctor_get(x_75, 1); lean_inc(x_81); -lean_dec_ref(x_77); +lean_dec_ref(x_75); x_82 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemDataFast___closed__5; x_83 = lean_string_append(x_79, x_82); x_84 = l_Nat_reprFast(x_80); @@ -1192,28 +1192,28 @@ x_86 = lean_string_append(x_85, x_82); x_87 = l_Nat_reprFast(x_81); x_88 = lean_string_append(x_86, x_87); lean_dec_ref(x_87); -if (lean_obj_tag(x_76) == 1) +if (lean_obj_tag(x_78) == 1) { lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_89 = lean_ctor_get(x_76, 0); +x_89 = lean_ctor_get(x_78, 0); lean_inc(x_89); -lean_dec_ref(x_76); +lean_dec_ref(x_78); x_90 = lean_string_append(x_88, x_82); x_91 = l_Nat_reprFast(x_89); x_92 = lean_string_append(x_90, x_91); lean_dec_ref(x_91); -x_44 = x_75; -x_45 = x_82; -x_46 = x_78; +x_44 = x_76; +x_45 = x_77; +x_46 = x_82; x_47 = x_92; goto block_74; } else { -lean_dec(x_76); -x_44 = x_75; -x_45 = x_82; -x_46 = x_78; +lean_dec(x_78); +x_44 = x_76; +x_45 = x_77; +x_46 = x_82; x_47 = x_88; goto block_74; } @@ -1250,10 +1250,10 @@ lean_object* x_109; lean_object* x_110; x_109 = lean_string_append(x_107, x_105); lean_dec_ref(x_105); x_110 = lean_string_append(x_109, x_106); -x_75 = x_99; -x_76 = x_98; -x_77 = x_97; -x_78 = x_104; +x_75 = x_97; +x_76 = x_104; +x_77 = x_99; +x_78 = x_98; x_79 = x_110; goto block_93; } @@ -1274,10 +1274,10 @@ x_115 = l_String_Slice_positions(x_114); lean_dec_ref(x_114); x_116 = l_WellFounded_opaqueFix_u2083___redArg(x_113, x_115, x_107, lean_box(0)); x_117 = lean_string_append(x_116, x_106); -x_75 = x_99; -x_76 = x_98; -x_77 = x_97; -x_78 = x_104; +x_75 = x_97; +x_76 = x_104; +x_77 = x_99; +x_78 = x_98; x_79 = x_117; goto block_93; } @@ -1774,14 +1774,14 @@ goto block_42; } block_78: { -if (lean_obj_tag(x_52) == 1) +if (lean_obj_tag(x_51) == 1) { lean_object* x_54; lean_object* x_55; -x_54 = lean_ctor_get(x_52, 0); +x_54 = lean_ctor_get(x_51, 0); lean_inc(x_54); -lean_dec_ref(x_52); -x_55 = lean_string_append(x_53, x_51); lean_dec_ref(x_51); +x_55 = lean_string_append(x_53, x_52); +lean_dec_ref(x_52); if (lean_obj_tag(x_54) == 0) { lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; @@ -1857,8 +1857,8 @@ goto block_46; } else { -lean_dec(x_52); -lean_dec_ref(x_51); +lean_dec_ref(x_52); +lean_dec(x_51); x_39 = x_53; goto block_42; } @@ -1866,11 +1866,11 @@ goto block_42; block_96: { 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_83 = lean_ctor_get(x_79, 0); +x_83 = lean_ctor_get(x_80, 0); lean_inc(x_83); -x_84 = lean_ctor_get(x_79, 1); +x_84 = lean_ctor_get(x_80, 1); lean_inc(x_84); -lean_dec_ref(x_79); +lean_dec_ref(x_80); x_85 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemDataFast___closed__5; x_86 = lean_string_append(x_82, x_85); x_87 = l_Nat_reprFast(x_83); @@ -1890,16 +1890,16 @@ x_93 = lean_string_append(x_91, x_85); x_94 = l_Nat_reprFast(x_92); x_95 = lean_string_append(x_93, x_94); lean_dec_ref(x_94); -x_51 = x_85; -x_52 = x_80; +x_51 = x_79; +x_52 = x_85; x_53 = x_95; goto block_78; } else { lean_dec(x_81); -x_51 = x_85; -x_52 = x_80; +x_51 = x_79; +x_52 = x_85; x_53 = x_91; goto block_78; } @@ -1932,10 +1932,10 @@ x_112 = lean_string_append(x_110, x_108); lean_dec_ref(x_108); x_113 = lean_string_append(x_112, x_109); lean_inc(x_102); -lean_inc(x_103); lean_inc_ref(x_101); -x_79 = x_101; -x_80 = x_103; +lean_inc(x_103); +x_79 = x_103; +x_80 = x_101; x_81 = x_102; x_82 = x_113; goto block_96; @@ -1956,10 +1956,10 @@ lean_dec_ref(x_108); lean_dec_ref(x_116); x_119 = lean_string_append(x_118, x_109); lean_inc(x_102); -lean_inc(x_103); lean_inc_ref(x_101); -x_79 = x_101; -x_80 = x_103; +lean_inc(x_103); +x_79 = x_103; +x_80 = x_101; x_81 = x_102; x_82 = x_119; goto block_96; @@ -2154,19 +2154,19 @@ goto block_219; { 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; uint8_t x_234; x_227 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressMarkupContentFast___closed__1; -x_228 = lean_string_append(x_225, x_227); +x_228 = lean_string_append(x_224, x_227); x_229 = lean_string_append(x_228, x_226); lean_dec_ref(x_226); x_230 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressMarkupContentFast___closed__2; x_231 = lean_string_append(x_229, x_230); x_232 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemDataFast___closed__1; x_233 = lean_string_append(x_231, x_232); -x_234 = l___private_Lean_Data_Json_Printer_0__Lean_Json_needEscape(x_224); +x_234 = l___private_Lean_Data_Json_Printer_0__Lean_Json_needEscape(x_225); if (x_234 == 0) { lean_object* x_235; lean_object* x_236; -x_235 = lean_string_append(x_233, x_224); -lean_dec_ref(x_224); +x_235 = lean_string_append(x_233, x_225); +lean_dec_ref(x_225); x_236 = lean_string_append(x_235, x_232); x_220 = x_236; goto block_223; @@ -2175,15 +2175,15 @@ else { lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; x_237 = lean_unsigned_to_nat(0u); -x_238 = lean_string_utf8_byte_size(x_224); -lean_inc_ref(x_224); +x_238 = lean_string_utf8_byte_size(x_225); +lean_inc_ref(x_225); x_239 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_239, 0, x_224); +lean_ctor_set(x_239, 0, x_225); lean_ctor_set(x_239, 1, x_237); lean_ctor_set(x_239, 2, x_238); x_240 = l_String_Slice_positions(x_239); -x_241 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemsFast_spec__0___redArg(x_239, x_224, x_240, x_233); -lean_dec_ref(x_224); +x_241 = l_WellFounded_opaqueFix_u2083___at___00__private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressItemsFast_spec__0___redArg(x_239, x_225, x_240, x_233); +lean_dec_ref(x_225); lean_dec_ref(x_239); x_242 = lean_string_append(x_241, x_232); x_220 = x_242; @@ -2207,8 +2207,8 @@ if (x_247 == 0) lean_object* x_251; x_251 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressMarkupContentFast___closed__3; lean_inc_ref(x_248); -x_224 = x_248; -x_225 = x_250; +x_224 = x_250; +x_225 = x_248; x_226 = x_251; goto block_243; } @@ -2217,8 +2217,8 @@ else lean_object* x_252; x_252 = l___private_Lean_Server_Completion_CompletionItemCompression_0__Lean_Lsp_ResolvableCompletionList_compressMarkupContentFast___closed__4; lean_inc_ref(x_248); -x_224 = x_248; -x_225 = x_250; +x_224 = x_250; +x_225 = x_248; x_226 = x_252; goto block_243; } diff --git a/stage0/stdlib/Lean/Server/FileWorker.c b/stage0/stdlib/Lean/Server/FileWorker.c index d9add6fd7839..5ecfe9d979fb 100644 --- a/stage0/stdlib/Lean/Server/FileWorker.c +++ b/stage0/stdlib/Lean/Server/FileWorker.c @@ -7156,10 +7156,10 @@ goto block_43; { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_7); +lean_ctor_set(x_9, 0, x_6); lean_ctor_set(x_9, 1, x_8); x_10 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_9); -x_11 = l_Std_Channel_Sync_send___redArg(x_6, x_10); +x_11 = l_Std_Channel_Sync_send___redArg(x_7, x_10); x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_11); lean_ctor_set(x_12, 1, x_4); @@ -7191,8 +7191,8 @@ if (lean_obj_tag(x_25) == 0) lean_object* x_26; lean_dec_ref(x_25); x_26 = lean_box(0); -x_6 = x_15; -x_7 = x_23; +x_6 = x_23; +x_7 = x_15; x_8 = x_26; goto block_13; } @@ -7202,8 +7202,8 @@ uint8_t x_27; x_27 = !lean_is_exclusive(x_25); if (x_27 == 0) { -x_6 = x_15; -x_7 = x_23; +x_6 = x_23; +x_7 = x_15; x_8 = x_25; goto block_13; } @@ -7215,8 +7215,8 @@ lean_inc(x_28); lean_dec(x_25); x_29 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_29, 0, x_28); -x_6 = x_15; -x_7 = x_23; +x_6 = x_23; +x_7 = x_15; x_8 = x_29; goto block_13; } @@ -7571,17 +7571,17 @@ return x_15; { lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 0, x_20); lean_ctor_set(x_23, 1, x_22); x_24 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_23); -x_25 = l_Std_Channel_Sync_send___redArg(x_19, x_24); -x_26 = lean_ctor_get_uint8(x_20, sizeof(void*)*2); -x_27 = lean_ctor_get(x_20, 0); +x_25 = l_Std_Channel_Sync_send___redArg(x_21, x_24); +x_26 = lean_ctor_get_uint8(x_19, sizeof(void*)*2); +x_27 = lean_ctor_get(x_19, 0); lean_inc_ref(x_27); -x_28 = lean_ctor_get_uint8(x_20, sizeof(void*)*2 + 1); -lean_dec_ref(x_20); +x_28 = lean_ctor_get_uint8(x_19, sizeof(void*)*2 + 1); +lean_dec_ref(x_19); x_29 = l___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_reportSnapshots_handleNode___closed__0; -x_6 = x_17; +x_6 = x_18; x_7 = x_29; x_8 = x_26; x_9 = x_27; @@ -7645,11 +7645,11 @@ lean_object* x_51; lean_dec_ref(x_50); lean_free_object(x_34); x_51 = lean_box(0); -x_17 = x_39; -x_18 = lean_box(0); -x_19 = x_47; -x_20 = x_37; -x_21 = x_48; +x_17 = lean_box(0); +x_18 = x_39; +x_19 = x_37; +x_20 = x_48; +x_21 = x_47; x_22 = x_51; goto block_30; } @@ -7660,11 +7660,11 @@ x_52 = lean_ctor_get(x_50, 0); lean_inc(x_52); lean_dec_ref(x_50); lean_ctor_set(x_34, 0, x_52); -x_17 = x_39; -x_18 = lean_box(0); -x_19 = x_47; -x_20 = x_37; -x_21 = x_48; +x_17 = lean_box(0); +x_18 = x_39; +x_19 = x_37; +x_20 = x_48; +x_21 = x_47; x_22 = x_34; goto block_30; } @@ -7719,11 +7719,11 @@ if (lean_obj_tag(x_64) == 0) lean_object* x_65; lean_dec_ref(x_64); x_65 = lean_box(0); -x_17 = x_53; -x_18 = lean_box(0); -x_19 = x_61; -x_20 = x_37; -x_21 = x_62; +x_17 = lean_box(0); +x_18 = x_53; +x_19 = x_37; +x_20 = x_62; +x_21 = x_61; x_22 = x_65; goto block_30; } @@ -7735,11 +7735,11 @@ lean_inc(x_66); lean_dec_ref(x_64); x_67 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_67, 0, x_66); -x_17 = x_53; -x_18 = lean_box(0); -x_19 = x_61; -x_20 = x_37; -x_21 = x_62; +x_17 = lean_box(0); +x_18 = x_53; +x_19 = x_37; +x_20 = x_62; +x_21 = x_61; x_22 = x_67; goto block_30; } @@ -9006,7 +9006,7 @@ goto block_91; { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 0, x_9); lean_ctor_set(x_12, 1, x_11); x_13 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_12); x_14 = l_Std_Channel_Sync_send___redArg(x_3, x_13); @@ -9029,8 +9029,8 @@ if (lean_obj_tag(x_25) == 0) lean_object* x_26; lean_dec_ref(x_25); x_26 = lean_box(0); -x_9 = lean_box(0); -x_10 = x_23; +x_9 = x_23; +x_10 = lean_box(0); x_11 = x_26; goto block_16; } @@ -9040,8 +9040,8 @@ uint8_t x_27; x_27 = !lean_is_exclusive(x_25); if (x_27 == 0) { -x_9 = lean_box(0); -x_10 = x_23; +x_9 = x_23; +x_10 = lean_box(0); x_11 = x_25; goto block_16; } @@ -9053,8 +9053,8 @@ lean_inc(x_28); lean_dec(x_25); x_29 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_29, 0, x_28); -x_9 = lean_box(0); -x_10 = x_23; +x_9 = x_23; +x_10 = lean_box(0); x_11 = x_29; goto block_16; } @@ -9092,7 +9092,7 @@ goto block_30; { lean_object* x_42; lean_object* x_43; lean_object* x_44; x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 0, x_38); lean_ctor_set(x_42, 1, x_41); x_43 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_42); lean_inc_ref(x_3); @@ -9106,13 +9106,13 @@ goto block_37; { lean_object* x_50; lean_object* x_51; lean_object* x_52; x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_47); +lean_ctor_set(x_50, 0, x_46); lean_ctor_set(x_50, 1, x_49); x_51 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_50); lean_inc_ref(x_3); x_52 = l_Std_Channel_send___redArg(x_3, x_51); lean_dec_ref(x_52); -x_31 = x_48; +x_31 = x_47; x_32 = lean_box(0); goto block_37; } @@ -9161,9 +9161,9 @@ x_78 = l_Lean_Json_toStructured_x3f___at___00__private_Lean_Server_FileWorker_0_ if (lean_obj_tag(x_78) == 0) { lean_dec_ref(x_78); -x_38 = lean_box(0); +x_38 = x_76; x_39 = x_72; -x_40 = x_76; +x_40 = lean_box(0); x_41 = x_57; goto block_45; } @@ -9173,9 +9173,9 @@ uint8_t x_79; x_79 = !lean_is_exclusive(x_78); if (x_79 == 0) { -x_38 = lean_box(0); +x_38 = x_76; x_39 = x_72; -x_40 = x_76; +x_40 = lean_box(0); x_41 = x_78; goto block_45; } @@ -9187,9 +9187,9 @@ lean_inc(x_80); lean_dec(x_78); x_81 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_81, 0, x_80); -x_38 = lean_box(0); +x_38 = x_76; x_39 = x_72; -x_40 = x_76; +x_40 = lean_box(0); x_41 = x_81; goto block_45; } @@ -9210,9 +9210,9 @@ x_86 = l_Lean_Json_toStructured_x3f___at___00__private_Lean_Server_FileWorker_0_ if (lean_obj_tag(x_86) == 0) { lean_dec_ref(x_86); -x_46 = lean_box(0); -x_47 = x_84; -x_48 = x_72; +x_46 = x_84; +x_47 = x_72; +x_48 = lean_box(0); x_49 = x_57; goto block_53; } @@ -9222,9 +9222,9 @@ uint8_t x_87; x_87 = !lean_is_exclusive(x_86); if (x_87 == 0) { -x_46 = lean_box(0); -x_47 = x_84; -x_48 = x_72; +x_46 = x_84; +x_47 = x_72; +x_48 = lean_box(0); x_49 = x_86; goto block_53; } @@ -9236,9 +9236,9 @@ lean_inc(x_88); lean_dec(x_86); x_89 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_89, 0, x_88); -x_46 = lean_box(0); -x_47 = x_84; -x_48 = x_72; +x_46 = x_84; +x_47 = x_72; +x_48 = lean_box(0); x_49 = x_89; goto block_53; } @@ -9706,7 +9706,7 @@ return x_4; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_setupImports(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_39; +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_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_39; x_20 = l_Lean_Server_FileWorker_setupImports___closed__0; x_21 = lean_st_ref_take(x_20); x_22 = 1; @@ -9777,15 +9777,15 @@ if (lean_is_scalar(x_44)) { x_54 = x_44; lean_ctor_set_tag(x_54, 1); } -lean_ctor_set(x_54, 0, x_49); +lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); x_55 = l_Lean_Server_FileWorker_OutputMessage_ofMsg(x_54); x_56 = l_Std_Channel_Sync_send___redArg(x_3, x_55); -switch (lean_obj_tag(x_52)) { +switch (lean_obj_tag(x_49)) { case 2: { lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; lean_object* x_62; lean_object* x_63; size_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -lean_dec_ref(x_50); +lean_dec_ref(x_51); lean_dec_ref(x_47); lean_dec_ref(x_46); lean_dec(x_2); @@ -9798,12 +9798,12 @@ x_61 = 0; x_62 = l_Lean_Server_FileWorker_setupImports___closed__5; x_63 = l_Lean_Server_FileWorker_setupImports___closed__6; x_64 = 5; -lean_inc(x_48); +lean_inc(x_50); x_65 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_65, 0, x_63); lean_ctor_set(x_65, 1, x_62); -lean_ctor_set(x_65, 2, x_48); -lean_ctor_set(x_65, 3, x_48); +lean_ctor_set(x_65, 2, x_50); +lean_ctor_set(x_65, 3, x_50); lean_ctor_set_usize(x_65, 4, x_64); x_66 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_66, 0, x_65); @@ -9828,16 +9828,16 @@ return x_71; case 3: { uint8_t x_72; -lean_dec_ref(x_50); +lean_dec_ref(x_51); lean_dec_ref(x_47); lean_dec_ref(x_46); lean_dec(x_2); lean_dec_ref(x_1); -x_72 = !lean_is_exclusive(x_52); +x_72 = !lean_is_exclusive(x_49); if (x_72 == 0) { lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint64_t x_77; lean_object* x_78; lean_object* x_79; size_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_73 = lean_ctor_get(x_52, 0); +x_73 = lean_ctor_get(x_49, 0); x_74 = l_Lean_Language_diagnosticsOfHeaderError(x_73, x_5); x_75 = l_Lean_Server_FileWorker_setupImports___closed__11; x_76 = lean_box(0); @@ -9845,12 +9845,12 @@ x_77 = 0; x_78 = l_Lean_Server_FileWorker_setupImports___closed__5; x_79 = l_Lean_Server_FileWorker_setupImports___closed__6; x_80 = 5; -lean_inc(x_48); +lean_inc(x_50); x_81 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_81, 0, x_79); lean_ctor_set(x_81, 1, x_78); -lean_ctor_set(x_81, 2, x_48); -lean_ctor_set(x_81, 3, x_48); +lean_ctor_set(x_81, 2, x_50); +lean_ctor_set(x_81, 3, x_50); lean_ctor_set_usize(x_81, 4, x_80); x_82 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_82, 0, x_81); @@ -9866,18 +9866,18 @@ x_85 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); lean_ctor_set(x_85, 2, x_76); -lean_ctor_set_tag(x_52, 0); -lean_ctor_set(x_52, 0, x_85); +lean_ctor_set_tag(x_49, 0); +lean_ctor_set(x_49, 0, x_85); x_86 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_86, 0, x_52); +lean_ctor_set(x_86, 0, x_49); return x_86; } else { lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint64_t x_91; lean_object* x_92; lean_object* x_93; size_t x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_87 = lean_ctor_get(x_52, 0); +x_87 = lean_ctor_get(x_49, 0); lean_inc(x_87); -lean_dec(x_52); +lean_dec(x_49); x_88 = l_Lean_Language_diagnosticsOfHeaderError(x_87, x_5); x_89 = l_Lean_Server_FileWorker_setupImports___closed__11; x_90 = lean_box(0); @@ -9885,12 +9885,12 @@ x_91 = 0; x_92 = l_Lean_Server_FileWorker_setupImports___closed__5; x_93 = l_Lean_Server_FileWorker_setupImports___closed__6; x_94 = 5; -lean_inc(x_48); +lean_inc(x_50); x_95 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_95, 0, x_93); lean_ctor_set(x_95, 1, x_92); -lean_ctor_set(x_95, 2, x_48); -lean_ctor_set(x_95, 3, x_48); +lean_ctor_set(x_95, 2, x_50); +lean_ctor_set(x_95, 3, x_50); lean_ctor_set_usize(x_95, 4, x_94); x_96 = lean_alloc_ctor(0, 1, 8); lean_ctor_set(x_96, 0, x_95); @@ -9916,21 +9916,21 @@ return x_101; default: { lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t 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; uint8_t x_117; -lean_dec(x_52); -lean_dec(x_48); +lean_dec(x_50); +lean_dec(x_49); lean_dec_ref(x_5); -x_102 = lean_ctor_get(x_50, 1); +x_102 = lean_ctor_get(x_51, 1); lean_inc(x_102); -x_103 = lean_ctor_get_uint8(x_50, sizeof(void*)*7); -x_104 = lean_ctor_get(x_50, 2); +x_103 = lean_ctor_get_uint8(x_51, sizeof(void*)*7); +x_104 = lean_ctor_get(x_51, 2); lean_inc(x_104); -x_105 = lean_ctor_get(x_50, 3); +x_105 = lean_ctor_get(x_51, 3); lean_inc(x_105); -x_106 = lean_ctor_get(x_50, 5); +x_106 = lean_ctor_get(x_51, 5); lean_inc_ref(x_106); -x_107 = lean_ctor_get(x_50, 6); +x_107 = lean_ctor_get(x_51, 6); lean_inc(x_107); -lean_dec_ref(x_50); +lean_dec_ref(x_51); x_108 = lean_ctor_get(x_1, 1); lean_inc(x_108); lean_dec_ref(x_1); @@ -9947,13 +9947,13 @@ x_116 = l_Lean_Option_set___at___00Lean_Server_FileWorker_setupImports_spec__1(x x_117 = lean_strict_or(x_103, x_110); if (lean_obj_tag(x_104) == 0) { -x_7 = x_117; -x_8 = x_105; -x_9 = lean_box(0); -x_10 = x_102; -x_11 = x_116; -x_12 = x_108; -x_13 = x_106; +x_7 = x_106; +x_8 = x_108; +x_9 = x_102; +x_10 = x_116; +x_11 = x_105; +x_12 = x_117; +x_13 = lean_box(0); x_14 = x_109; goto block_19; } @@ -9964,13 +9964,13 @@ lean_dec_ref(x_109); x_118 = lean_ctor_get(x_104, 0); lean_inc(x_118); lean_dec_ref(x_104); -x_7 = x_117; -x_8 = x_105; -x_9 = lean_box(0); -x_10 = x_102; -x_11 = x_116; -x_12 = x_108; -x_13 = x_106; +x_7 = x_106; +x_8 = x_108; +x_9 = x_102; +x_10 = x_116; +x_11 = x_105; +x_12 = x_117; +x_13 = lean_box(0); x_14 = x_118; goto block_19; } @@ -10001,11 +10001,11 @@ if (lean_obj_tag(x_133) == 0) lean_object* x_134; lean_dec_ref(x_133); x_134 = lean_box(0); -x_48 = x_128; -x_49 = x_131; -x_50 = x_120; -x_51 = lean_box(0); -x_52 = x_122; +x_48 = lean_box(0); +x_49 = x_120; +x_50 = x_128; +x_51 = x_122; +x_52 = x_131; x_53 = x_134; goto block_119; } @@ -10015,11 +10015,11 @@ uint8_t x_135; x_135 = !lean_is_exclusive(x_133); if (x_135 == 0) { -x_48 = x_128; -x_49 = x_131; -x_50 = x_120; -x_51 = lean_box(0); -x_52 = x_122; +x_48 = lean_box(0); +x_49 = x_120; +x_50 = x_128; +x_51 = x_122; +x_52 = x_131; x_53 = x_133; goto block_119; } @@ -10031,11 +10031,11 @@ lean_inc(x_136); lean_dec(x_133); x_137 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_137, 0, x_136); -x_48 = x_128; -x_49 = x_131; -x_50 = x_120; -x_51 = lean_box(0); -x_52 = x_122; +x_48 = lean_box(0); +x_49 = x_120; +x_50 = x_128; +x_51 = x_122; +x_52 = x_131; x_53 = x_137; goto block_119; } @@ -10058,7 +10058,7 @@ lean_dec_ref(x_146); x_147 = lean_box(0); x_120 = x_139; x_121 = x_144; -x_122 = x_141; +x_122 = x_140; x_123 = lean_box(0); x_124 = x_147; goto block_138; @@ -10071,7 +10071,7 @@ if (x_148 == 0) { x_120 = x_139; x_121 = x_144; -x_122 = x_141; +x_122 = x_140; x_123 = lean_box(0); x_124 = x_146; goto block_138; @@ -10086,7 +10086,7 @@ x_150 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_150, 0, x_149); x_120 = x_139; x_121 = x_144; -x_122 = x_141; +x_122 = x_140; x_123 = lean_box(0); x_124 = x_150; goto block_138; @@ -10119,9 +10119,9 @@ lean_dec(x_21); x_159 = lean_ctor_get(x_157, 1); lean_inc_ref(x_159); lean_dec(x_157); -x_139 = x_159; -x_140 = lean_box(0); -x_141 = x_158; +x_139 = x_158; +x_140 = x_159; +x_141 = lean_box(0); x_142 = x_22; goto block_151; } @@ -10134,9 +10134,9 @@ lean_dec(x_21); x_160 = lean_ctor_get(x_157, 1); lean_inc_ref(x_160); lean_dec(x_157); -x_139 = x_160; -x_140 = lean_box(0); -x_141 = x_158; +x_139 = x_158; +x_140 = x_160; +x_141 = lean_box(0); x_142 = x_22; goto block_151; } @@ -10148,9 +10148,9 @@ lean_inc_ref(x_161); lean_dec(x_157); x_162 = lean_unbox(x_21); lean_dec(x_21); -x_139 = x_161; -x_140 = lean_box(0); -x_141 = x_158; +x_139 = x_158; +x_140 = x_161; +x_141 = lean_box(0); x_142 = x_162; goto block_151; } @@ -10239,13 +10239,13 @@ goto block_38; uint32_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; x_15 = 0; x_16 = lean_alloc_ctor(0, 6, 5); -lean_ctor_set(x_16, 0, x_12); -lean_ctor_set(x_16, 1, x_10); +lean_ctor_set(x_16, 0, x_8); +lean_ctor_set(x_16, 1, x_9); lean_ctor_set(x_16, 2, x_14); -lean_ctor_set(x_16, 3, x_11); -lean_ctor_set(x_16, 4, x_8); -lean_ctor_set(x_16, 5, x_13); -lean_ctor_set_uint8(x_16, sizeof(void*)*6 + 4, x_7); +lean_ctor_set(x_16, 3, x_10); +lean_ctor_set(x_16, 4, x_11); +lean_ctor_set(x_16, 5, x_7); +lean_ctor_set_uint8(x_16, sizeof(void*)*6 + 4, x_12); lean_ctor_set_uint32(x_16, sizeof(void*)*6, x_15); x_17 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -14175,9 +14175,9 @@ goto block_54; block_47: { lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_nat_add(x_41, x_43); +x_44 = lean_nat_add(x_42, x_43); lean_dec(x_43); -lean_dec(x_41); +lean_dec(x_42); if (lean_is_scalar(x_38)) { x_45 = lean_alloc_ctor(0, 5, 0); } else { @@ -14196,7 +14196,7 @@ if (lean_is_scalar(x_28)) { lean_ctor_set(x_46, 0, x_40); lean_ctor_set(x_46, 1, x_30); lean_ctor_set(x_46, 2, x_31); -lean_ctor_set(x_46, 3, x_42); +lean_ctor_set(x_46, 3, x_41); lean_ctor_set(x_46, 4, x_45); return x_46; } @@ -14222,8 +14222,8 @@ if (lean_obj_tag(x_33) == 0) lean_object* x_52; x_52 = lean_ctor_get(x_33, 0); lean_inc(x_52); -x_41 = x_51; -x_42 = x_50; +x_41 = x_50; +x_42 = x_51; x_43 = x_52; goto block_47; } @@ -14231,8 +14231,8 @@ else { lean_object* x_53; x_53 = lean_unsigned_to_nat(0u); -x_41 = x_51; -x_42 = x_50; +x_41 = x_50; +x_42 = x_51; x_43 = x_53; goto block_47; } @@ -14649,9 +14649,9 @@ goto block_155; block_147: { lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_144 = lean_nat_add(x_141, x_143); +x_144 = lean_nat_add(x_142, x_143); lean_dec(x_143); -lean_dec(x_141); +lean_dec(x_142); if (lean_is_scalar(x_138)) { x_145 = lean_alloc_ctor(0, 5, 0); } else { @@ -14670,7 +14670,7 @@ if (lean_is_scalar(x_128)) { lean_ctor_set(x_146, 0, x_140); lean_ctor_set(x_146, 1, x_131); lean_ctor_set(x_146, 2, x_132); -lean_ctor_set(x_146, 3, x_142); +lean_ctor_set(x_146, 3, x_141); lean_ctor_set(x_146, 4, x_145); return x_146; } @@ -14696,8 +14696,8 @@ if (lean_obj_tag(x_134) == 0) lean_object* x_153; x_153 = lean_ctor_get(x_134, 0); lean_inc(x_153); -x_141 = x_152; -x_142 = x_151; +x_141 = x_151; +x_142 = x_152; x_143 = x_153; goto block_147; } @@ -14705,8 +14705,8 @@ else { lean_object* x_154; x_154 = lean_unsigned_to_nat(0u); -x_141 = x_152; -x_142 = x_151; +x_141 = x_151; +x_142 = x_152; x_143 = x_154; goto block_147; } @@ -16717,14 +16717,14 @@ goto block_14; } block_19: { -if (x_17 == 0) +if (x_18 == 0) { x_15 = x_11; goto block_16; } else { -if (x_18 == 0) +if (x_17 == 0) { x_15 = x_11; goto block_16; @@ -16759,8 +16759,8 @@ x_31 = lean_nat_dec_le(x_27, x_23); if (x_31 == 0) { lean_dec(x_23); -x_17 = x_30; -x_18 = x_29; +x_17 = x_29; +x_18 = x_30; goto block_19; } else @@ -16770,8 +16770,8 @@ x_32 = lean_nat_dec_lt(x_23, x_28); lean_dec(x_23); if (x_32 == 0) { -x_17 = x_30; -x_18 = x_29; +x_17 = x_29; +x_18 = x_30; goto block_19; } else @@ -18251,14 +18251,14 @@ if (lean_is_scalar(x_14)) { x_26 = x_14; } lean_ctor_set(x_26, 0, x_15); -lean_ctor_set(x_26, 1, x_19); +lean_ctor_set(x_26, 1, x_16); lean_ctor_set(x_26, 2, x_23); -lean_ctor_set(x_26, 3, x_17); -lean_ctor_set(x_26, 4, x_22); -lean_ctor_set(x_26, 5, x_18); -lean_ctor_set(x_26, 6, x_21); +lean_ctor_set(x_26, 3, x_19); +lean_ctor_set(x_26, 4, x_18); +lean_ctor_set(x_26, 5, x_22); +lean_ctor_set(x_26, 6, x_17); lean_ctor_set(x_26, 7, x_20); -lean_ctor_set(x_26, 8, x_16); +lean_ctor_set(x_26, 8, x_21); lean_ctor_set(x_26, 9, x_24); lean_ctor_set(x_26, 10, x_13); x_27 = l_Lean_Widget_instToJsonRpcEncodablePacket_toJson_00___x40_Lean_Widget_InteractiveDiagnostic_3833933514____hygCtx___hyg_123_(x_26); @@ -18274,13 +18274,13 @@ if (lean_obj_tag(x_12) == 0) { lean_object* x_39; x_39 = lean_box(0); -x_16 = x_37; -x_17 = x_30; -x_18 = x_31; +x_16 = x_30; +x_17 = x_31; +x_18 = x_33; x_19 = x_32; -x_20 = x_33; -x_21 = x_35; -x_22 = x_34; +x_20 = x_34; +x_21 = x_37; +x_22 = x_35; x_23 = x_36; x_24 = x_39; x_25 = x_38; @@ -18304,13 +18304,13 @@ lean_inc(x_46); lean_dec_ref(x_44); x_47 = l_Array_toJson___at___00Lean_Server_FileWorker_handlePreRequestSpecialCases_x3f_spec__6(x_45); lean_ctor_set(x_12, 0, x_47); -x_16 = x_37; -x_17 = x_30; -x_18 = x_31; +x_16 = x_30; +x_17 = x_31; +x_18 = x_33; x_19 = x_32; -x_20 = x_33; -x_21 = x_35; -x_22 = x_34; +x_20 = x_34; +x_21 = x_37; +x_22 = x_35; x_23 = x_36; x_24 = x_12; x_25 = x_46; @@ -18333,13 +18333,13 @@ lean_dec_ref(x_51); x_54 = l_Array_toJson___at___00Lean_Server_FileWorker_handlePreRequestSpecialCases_x3f_spec__6(x_52); x_55 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_55, 0, x_54); -x_16 = x_37; -x_17 = x_30; -x_18 = x_31; +x_16 = x_30; +x_17 = x_31; +x_18 = x_33; x_19 = x_32; -x_20 = x_33; -x_21 = x_35; -x_22 = x_34; +x_20 = x_34; +x_21 = x_37; +x_22 = x_35; x_23 = x_36; x_24 = x_55; x_25 = x_53; @@ -18355,10 +18355,10 @@ lean_object* x_65; x_65 = lean_box(0); x_30 = x_57; x_31 = x_58; -x_32 = x_59; -x_33 = x_63; -x_34 = x_61; -x_35 = x_60; +x_32 = x_60; +x_33 = x_59; +x_34 = x_63; +x_35 = x_61; x_36 = x_62; x_37 = x_65; x_38 = x_64; @@ -18384,10 +18384,10 @@ x_73 = l_Array_toJson___at___00Lean_Server_FileWorker_handlePreRequestSpecialCas lean_ctor_set(x_11, 0, x_73); x_30 = x_57; x_31 = x_58; -x_32 = x_59; -x_33 = x_63; -x_34 = x_61; -x_35 = x_60; +x_32 = x_60; +x_33 = x_59; +x_34 = x_63; +x_35 = x_61; x_36 = x_62; x_37 = x_11; x_38 = x_72; @@ -18412,10 +18412,10 @@ x_81 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_81, 0, x_80); x_30 = x_57; x_31 = x_58; -x_32 = x_59; -x_33 = x_63; -x_34 = x_61; -x_35 = x_60; +x_32 = x_60; +x_33 = x_59; +x_34 = x_63; +x_35 = x_61; x_36 = x_62; x_37 = x_81; x_38 = x_79; @@ -18439,10 +18439,10 @@ if (lean_obj_tag(x_10) == 0) lean_object* x_94; x_94 = lean_box(0); x_57 = x_83; -x_58 = x_87; -x_59 = x_84; -x_60 = x_93; -x_61 = x_85; +x_58 = x_93; +x_59 = x_85; +x_60 = x_84; +x_61 = x_87; x_62 = x_86; x_63 = x_94; x_64 = x_92; @@ -18467,10 +18467,10 @@ lean_dec_ref(x_99); x_102 = l_Array_toJson___at___00Lean_Server_FileWorker_handlePreRequestSpecialCases_x3f_spec__6(x_100); lean_ctor_set(x_10, 0, x_102); x_57 = x_83; -x_58 = x_87; -x_59 = x_84; -x_60 = x_93; -x_61 = x_85; +x_58 = x_93; +x_59 = x_85; +x_60 = x_84; +x_61 = x_87; x_62 = x_86; x_63 = x_10; x_64 = x_101; @@ -18494,10 +18494,10 @@ x_109 = l_Array_toJson___at___00Lean_Server_FileWorker_handlePreRequestSpecialCa x_110 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_110, 0, x_109); x_57 = x_83; -x_58 = x_87; -x_59 = x_84; -x_60 = x_93; -x_61 = x_85; +x_58 = x_93; +x_59 = x_85; +x_60 = x_84; +x_61 = x_87; x_62 = x_86; x_63 = x_110; x_64 = x_108; @@ -18576,8 +18576,8 @@ if (lean_obj_tag(x_7) == 0) { lean_object* x_136; x_136 = lean_box(0); -x_112 = x_134; -x_113 = x_132; +x_112 = x_132; +x_113 = x_134; x_114 = x_133; x_115 = x_136; x_116 = x_135; @@ -18600,8 +18600,8 @@ x_139 = lean_ctor_get(x_137, 0); x_140 = l_Lean_JsonNumber_fromInt(x_139); lean_ctor_set_tag(x_137, 2); lean_ctor_set(x_137, 0, x_140); -x_125 = x_134; -x_126 = x_132; +x_125 = x_132; +x_126 = x_134; x_127 = x_133; x_128 = x_137; x_129 = x_135; @@ -18616,8 +18616,8 @@ lean_dec(x_137); x_142 = l_Lean_JsonNumber_fromInt(x_141); x_143 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_143, 0, x_142); -x_125 = x_134; -x_126 = x_132; +x_125 = x_132; +x_126 = x_134; x_127 = x_133; x_128 = x_143; x_129 = x_135; @@ -18631,8 +18631,8 @@ x_144 = !lean_is_exclusive(x_137); if (x_144 == 0) { lean_ctor_set_tag(x_137, 3); -x_125 = x_134; -x_126 = x_132; +x_125 = x_132; +x_126 = x_134; x_127 = x_133; x_128 = x_137; x_129 = x_135; @@ -18646,8 +18646,8 @@ lean_inc(x_145); lean_dec(x_137); x_146 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_146, 0, x_145); -x_125 = x_134; -x_126 = x_132; +x_125 = x_132; +x_126 = x_134; x_127 = x_133; x_128 = x_146; x_129 = x_135; @@ -20683,7 +20683,7 @@ if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_dec_ref(x_22); -x_23 = l_Lean_Server_FileWorker_handleUnknownIdentifierCodeAction(x_2, x_1, x_11, x_13, x_5); +x_23 = l_Lean_Server_FileWorker_handleUnknownIdentifierCodeAction(x_2, x_1, x_12, x_13, x_5); if (lean_obj_tag(x_23) == 0) { uint8_t x_24; @@ -20761,7 +20761,7 @@ uint8_t x_39; lean_dec(x_18); lean_free_object(x_4); lean_dec_ref(x_13); -lean_dec_ref(x_11); +lean_dec_ref(x_12); lean_dec(x_10); lean_dec_ref(x_5); lean_dec(x_2); @@ -20789,7 +20789,7 @@ uint8_t x_42; lean_dec(x_18); lean_free_object(x_4); lean_dec_ref(x_13); -lean_dec_ref(x_11); +lean_dec_ref(x_12); lean_dec(x_10); lean_dec_ref(x_5); lean_dec(x_2); @@ -20830,7 +20830,7 @@ if (lean_obj_tag(x_49) == 0) { lean_object* x_50; lean_dec_ref(x_49); -x_50 = l_Lean_Server_FileWorker_handleUnknownIdentifierCodeAction(x_2, x_1, x_11, x_13, x_5); +x_50 = l_Lean_Server_FileWorker_handleUnknownIdentifierCodeAction(x_2, x_1, x_12, x_13, x_5); if (lean_obj_tag(x_50) == 0) { lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; @@ -20894,7 +20894,7 @@ else lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec(x_45); lean_dec_ref(x_13); -lean_dec_ref(x_11); +lean_dec_ref(x_12); lean_dec(x_10); lean_dec_ref(x_5); lean_dec(x_2); @@ -20922,7 +20922,7 @@ else lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_dec(x_45); lean_dec_ref(x_13); -lean_dec_ref(x_11); +lean_dec_ref(x_12); lean_dec(x_10); lean_dec_ref(x_5); lean_dec(x_2); @@ -20951,7 +20951,7 @@ else lean_object* x_68; lean_dec_ref(x_14); lean_dec_ref(x_13); -lean_dec_ref(x_11); +lean_dec_ref(x_12); lean_dec(x_10); lean_dec_ref(x_5); lean_dec(x_2); @@ -20987,8 +20987,8 @@ if (x_80 == 0) { lean_object* x_81; x_81 = l_Lean_Server_FileWorker_handlePostRequestSpecialCases___lam__0___closed__0; -x_11 = x_75; -x_12 = lean_box(0); +x_11 = lean_box(0); +x_12 = x_75; x_13 = x_81; goto block_69; } @@ -20996,8 +20996,8 @@ else { lean_object* x_82; x_82 = l_Lean_Server_FileWorker_handlePostRequestSpecialCases___lam__0___closed__1; -x_11 = x_75; -x_12 = lean_box(0); +x_11 = lean_box(0); +x_12 = x_75; x_13 = x_82; goto block_69; } @@ -22414,9 +22414,9 @@ goto block_53; block_45: { lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_nat_add(x_40, x_41); +x_42 = lean_nat_add(x_39, x_41); lean_dec(x_41); -lean_dec(x_40); +lean_dec(x_39); if (lean_is_scalar(x_36)) { x_43 = lean_alloc_ctor(0, 5, 0); } else { @@ -22435,7 +22435,7 @@ if (lean_is_scalar(x_26)) { lean_ctor_set(x_44, 0, x_38); lean_ctor_set(x_44, 1, x_29); lean_ctor_set(x_44, 2, x_30); -lean_ctor_set(x_44, 3, x_39); +lean_ctor_set(x_44, 3, x_40); lean_ctor_set(x_44, 4, x_43); return x_44; } @@ -22462,8 +22462,8 @@ if (lean_obj_tag(x_32) == 0) lean_object* x_51; x_51 = lean_ctor_get(x_32, 0); lean_inc(x_51); -x_39 = x_49; -x_40 = x_50; +x_39 = x_50; +x_40 = x_49; x_41 = x_51; goto block_45; } @@ -22471,8 +22471,8 @@ else { lean_object* x_52; x_52 = lean_unsigned_to_nat(0u); -x_39 = x_49; -x_40 = x_50; +x_39 = x_50; +x_40 = x_49; x_41 = x_52; goto block_45; } @@ -23016,9 +23016,9 @@ goto block_186; block_179: { lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_176 = lean_nat_add(x_174, x_175); +x_176 = lean_nat_add(x_173, x_175); lean_dec(x_175); -lean_dec(x_174); +lean_dec(x_173); if (lean_is_scalar(x_170)) { x_177 = lean_alloc_ctor(0, 5, 0); } else { @@ -23037,7 +23037,7 @@ if (lean_is_scalar(x_160)) { lean_ctor_set(x_178, 0, x_172); lean_ctor_set(x_178, 1, x_162); lean_ctor_set(x_178, 2, x_163); -lean_ctor_set(x_178, 3, x_173); +lean_ctor_set(x_178, 3, x_174); lean_ctor_set(x_178, 4, x_177); return x_178; } @@ -23063,8 +23063,8 @@ if (lean_obj_tag(x_165) == 0) lean_object* x_184; x_184 = lean_ctor_get(x_165, 0); lean_inc(x_184); -x_173 = x_182; -x_174 = x_183; +x_173 = x_183; +x_174 = x_182; x_175 = x_184; goto block_179; } @@ -23072,8 +23072,8 @@ else { lean_object* x_185; x_185 = lean_unsigned_to_nat(0u); -x_173 = x_182; -x_174 = x_183; +x_173 = x_183; +x_174 = x_182; x_175 = x_185; goto block_179; } @@ -23562,9 +23562,9 @@ goto block_305; block_297: { lean_object* x_288; lean_object* x_289; uint8_t x_290; -x_288 = lean_nat_add(x_285, x_287); +x_288 = lean_nat_add(x_286, x_287); lean_dec(x_287); -lean_dec(x_285); +lean_dec(x_286); lean_inc_ref(x_257); if (lean_is_scalar(x_282)) { x_289 = lean_alloc_ctor(0, 5, 0); @@ -23591,7 +23591,7 @@ lean_dec(x_294); x_295 = lean_ctor_get(x_257, 0); lean_dec(x_295); lean_ctor_set(x_257, 4, x_289); -lean_ctor_set(x_257, 3, x_286); +lean_ctor_set(x_257, 3, x_285); lean_ctor_set(x_257, 2, x_276); lean_ctor_set(x_257, 1, x_275); lean_ctor_set(x_257, 0, x_284); @@ -23605,7 +23605,7 @@ x_296 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_296, 0, x_284); lean_ctor_set(x_296, 1, x_275); lean_ctor_set(x_296, 2, x_276); -lean_ctor_set(x_296, 3, x_286); +lean_ctor_set(x_296, 3, x_285); lean_ctor_set(x_296, 4, x_289); return x_296; } @@ -23632,8 +23632,8 @@ if (lean_obj_tag(x_278) == 0) lean_object* x_303; x_303 = lean_ctor_get(x_278, 0); lean_inc(x_303); -x_285 = x_302; -x_286 = x_301; +x_285 = x_301; +x_286 = x_302; x_287 = x_303; goto block_297; } @@ -23641,8 +23641,8 @@ else { lean_object* x_304; x_304 = lean_unsigned_to_nat(0u); -x_285 = x_302; -x_286 = x_301; +x_285 = x_301; +x_286 = x_302; x_287 = x_304; goto block_297; } @@ -23728,9 +23728,9 @@ goto block_340; block_332: { lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; -x_328 = lean_nat_add(x_325, x_327); +x_328 = lean_nat_add(x_326, x_327); lean_dec(x_327); -lean_dec(x_325); +lean_dec(x_326); lean_inc_ref(x_257); if (lean_is_scalar(x_322)) { x_329 = lean_alloc_ctor(0, 5, 0); @@ -23761,7 +23761,7 @@ if (lean_is_scalar(x_330)) { lean_ctor_set(x_331, 0, x_324); lean_ctor_set(x_331, 1, x_315); lean_ctor_set(x_331, 2, x_316); -lean_ctor_set(x_331, 3, x_326); +lean_ctor_set(x_331, 3, x_325); lean_ctor_set(x_331, 4, x_329); return x_331; } @@ -23787,8 +23787,8 @@ if (lean_obj_tag(x_318) == 0) lean_object* x_338; x_338 = lean_ctor_get(x_318, 0); lean_inc(x_338); -x_325 = x_337; -x_326 = x_336; +x_325 = x_336; +x_326 = x_337; x_327 = x_338; goto block_332; } @@ -23796,8 +23796,8 @@ else { lean_object* x_339; x_339 = lean_unsigned_to_nat(0u); -x_325 = x_337; -x_326 = x_336; +x_325 = x_336; +x_326 = x_337; x_327 = x_339; goto block_332; } @@ -24266,9 +24266,9 @@ goto block_451; block_444: { lean_object* x_441; lean_object* x_442; lean_object* x_443; -x_441 = lean_nat_add(x_439, x_440); +x_441 = lean_nat_add(x_438, x_440); lean_dec(x_440); -lean_dec(x_439); +lean_dec(x_438); if (lean_is_scalar(x_435)) { x_442 = lean_alloc_ctor(0, 5, 0); } else { @@ -24287,7 +24287,7 @@ if (lean_is_scalar(x_425)) { lean_ctor_set(x_443, 0, x_437); lean_ctor_set(x_443, 1, x_427); lean_ctor_set(x_443, 2, x_428); -lean_ctor_set(x_443, 3, x_438); +lean_ctor_set(x_443, 3, x_439); lean_ctor_set(x_443, 4, x_442); return x_443; } @@ -24313,8 +24313,8 @@ if (lean_obj_tag(x_430) == 0) lean_object* x_449; x_449 = lean_ctor_get(x_430, 0); lean_inc(x_449); -x_438 = x_447; -x_439 = x_448; +x_438 = x_448; +x_439 = x_447; x_440 = x_449; goto block_444; } @@ -24322,8 +24322,8 @@ else { lean_object* x_450; x_450 = lean_unsigned_to_nat(0u); -x_438 = x_447; -x_439 = x_448; +x_438 = x_448; +x_439 = x_447; x_440 = x_450; goto block_444; } @@ -27852,7 +27852,7 @@ goto block_167; { 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; x_135 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 0, x_131); lean_ctor_set(x_135, 1, x_134); x_136 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__8; x_137 = lean_alloc_ctor(3, 1, 0); @@ -27873,13 +27873,13 @@ lean_dec(x_130); x_144 = l_List_appendTR___redArg(x_141, x_143); x_145 = l_Lean_Json_mkObj(x_144); x_146 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_146, 0, x_131); +lean_ctor_set(x_146, 0, x_132); lean_ctor_set(x_146, 1, x_145); x_147 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_147, 0, x_146); lean_ctor_set(x_147, 1, x_139); x_148 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_148, 0, x_132); +lean_ctor_set(x_148, 0, x_133); lean_ctor_set(x_148, 1, x_147); x_68 = x_148; goto block_77; @@ -27897,9 +27897,9 @@ case 0: { lean_object* x_155; x_155 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__15; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_155; goto block_149; } @@ -27907,9 +27907,9 @@ case 1: { lean_object* x_156; x_156 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__19; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_156; goto block_149; } @@ -27917,9 +27917,9 @@ case 2: { lean_object* x_157; x_157 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__23; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_157; goto block_149; } @@ -27927,9 +27927,9 @@ case 3: { lean_object* x_158; x_158 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__27; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_158; goto block_149; } @@ -27937,9 +27937,9 @@ case 4: { lean_object* x_159; x_159 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__31; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_159; goto block_149; } @@ -27947,9 +27947,9 @@ case 5: { lean_object* x_160; x_160 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__35; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_160; goto block_149; } @@ -27957,9 +27957,9 @@ case 6: { lean_object* x_161; x_161 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__39; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_161; goto block_149; } @@ -27967,9 +27967,9 @@ case 7: { lean_object* x_162; x_162 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__43; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_162; goto block_149; } @@ -27977,9 +27977,9 @@ case 8: { lean_object* x_163; x_163 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__47; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_163; goto block_149; } @@ -27987,9 +27987,9 @@ case 9: { lean_object* x_164; x_164 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__51; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_164; goto block_149; } @@ -27997,9 +27997,9 @@ case 10: { lean_object* x_165; x_165 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__55; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_165; goto block_149; } @@ -28007,9 +28007,9 @@ goto block_149; { lean_object* x_166; x_166 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__59; -x_131 = x_153; -x_132 = x_152; -x_133 = x_154; +x_131 = x_154; +x_132 = x_153; +x_133 = x_152; x_134 = x_166; goto block_149; } @@ -28431,7 +28431,7 @@ return x_36; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_86; uint8_t x_87; lean_object* x_88; uint8_t x_94; lean_object* x_102; lean_object* x_103; +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; 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; uint8_t x_69; lean_object* x_70; lean_object* x_71; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_86; uint8_t x_87; lean_object* x_88; uint8_t x_94; lean_object* x_102; lean_object* x_103; x_37 = lean_ctor_get(x_24, 0); lean_inc(x_37); lean_dec_ref(x_24); @@ -28473,13 +28473,13 @@ goto block_101; { lean_object* x_44; lean_object* x_45; lean_object* x_46; x_44 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_44, 0, x_40); -lean_ctor_set(x_44, 1, x_38); -lean_ctor_set(x_44, 2, x_41); -lean_ctor_set(x_44, 3, x_39); +lean_ctor_set(x_44, 0, x_39); +lean_ctor_set(x_44, 1, x_41); +lean_ctor_set(x_44, 2, x_38); +lean_ctor_set(x_44, 3, x_42); lean_ctor_set(x_44, 4, x_37); lean_ctor_set(x_44, 5, x_43); -lean_ctor_set_uint8(x_44, sizeof(void*)*6, x_42); +lean_ctor_set_uint8(x_44, sizeof(void*)*6, x_40); if (lean_is_scalar(x_11)) { x_45 = lean_alloc_ctor(0, 3, 0); } else { @@ -28498,46 +28498,46 @@ return x_46; } block_58: { -if (lean_obj_tag(x_49) == 0) +if (lean_obj_tag(x_50) == 0) { lean_object* x_54; -lean_dec_ref(x_49); +lean_dec_ref(x_50); x_54 = lean_box(0); x_38 = x_48; -x_39 = x_53; -x_40 = x_50; -x_41 = x_51; -x_42 = x_52; +x_39 = x_49; +x_40 = x_51; +x_41 = x_52; +x_42 = x_53; x_43 = x_54; goto block_47; } else { uint8_t x_55; -x_55 = !lean_is_exclusive(x_49); +x_55 = !lean_is_exclusive(x_50); if (x_55 == 0) { x_38 = x_48; -x_39 = x_53; -x_40 = x_50; -x_41 = x_51; -x_42 = x_52; -x_43 = x_49; +x_39 = x_49; +x_40 = x_51; +x_41 = x_52; +x_42 = x_53; +x_43 = x_50; goto block_47; } else { lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_49, 0); +x_56 = lean_ctor_get(x_50, 0); lean_inc(x_56); -lean_dec(x_49); +lean_dec(x_50); x_57 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_57, 0, x_56); x_38 = x_48; -x_39 = x_53; -x_40 = x_50; -x_41 = x_51; -x_42 = x_52; +x_39 = x_49; +x_40 = x_51; +x_41 = x_52; +x_42 = x_53; x_43 = x_57; goto block_47; } @@ -28550,10 +28550,10 @@ if (lean_obj_tag(x_66) == 0) lean_object* x_72; lean_dec_ref(x_66); x_72 = lean_box(0); -x_48 = x_67; -x_49 = x_68; -x_50 = x_69; -x_51 = x_71; +x_48 = x_71; +x_49 = x_67; +x_50 = x_68; +x_51 = x_69; x_52 = x_70; x_53 = x_72; goto block_58; @@ -28564,10 +28564,10 @@ uint8_t x_73; x_73 = !lean_is_exclusive(x_66); if (x_73 == 0) { -x_48 = x_67; -x_49 = x_68; -x_50 = x_69; -x_51 = x_71; +x_48 = x_71; +x_49 = x_67; +x_50 = x_68; +x_51 = x_69; x_52 = x_70; x_53 = x_66; goto block_58; @@ -28580,10 +28580,10 @@ lean_inc(x_74); lean_dec(x_66); x_75 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_75, 0, x_74); -x_48 = x_67; -x_49 = x_68; -x_50 = x_69; -x_51 = x_71; +x_48 = x_71; +x_49 = x_67; +x_50 = x_68; +x_51 = x_69; x_52 = x_70; x_53 = x_75; goto block_58; @@ -28597,10 +28597,10 @@ if (lean_obj_tag(x_64) == 0) lean_object* x_81; lean_dec_ref(x_64); x_81 = lean_box(0); -x_67 = x_80; -x_68 = x_77; -x_69 = x_78; -x_70 = x_79; +x_67 = x_77; +x_68 = x_78; +x_69 = x_79; +x_70 = x_80; x_71 = x_81; goto block_76; } @@ -28610,10 +28610,10 @@ uint8_t x_82; x_82 = !lean_is_exclusive(x_64); if (x_82 == 0) { -x_67 = x_80; -x_68 = x_77; -x_69 = x_78; -x_70 = x_79; +x_67 = x_77; +x_68 = x_78; +x_69 = x_79; +x_70 = x_80; x_71 = x_64; goto block_76; } @@ -28625,10 +28625,10 @@ lean_inc(x_83); lean_dec(x_64); x_84 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_84, 0, x_83); -x_67 = x_80; -x_68 = x_77; -x_69 = x_78; -x_70 = x_79; +x_67 = x_77; +x_68 = x_78; +x_69 = x_79; +x_70 = x_80; x_71 = x_84; goto block_76; } @@ -28641,8 +28641,8 @@ if (lean_obj_tag(x_62) == 0) lean_object* x_89; lean_dec_ref(x_62); x_89 = lean_box(0); -x_77 = x_86; -x_78 = x_88; +x_77 = x_88; +x_78 = x_86; x_79 = x_87; x_80 = x_89; goto block_85; @@ -28653,8 +28653,8 @@ uint8_t x_90; x_90 = !lean_is_exclusive(x_62); if (x_90 == 0) { -x_77 = x_86; -x_78 = x_88; +x_77 = x_88; +x_78 = x_86; x_79 = x_87; x_80 = x_62; goto block_85; @@ -28667,8 +28667,8 @@ lean_inc(x_91); lean_dec(x_62); x_92 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_92, 0, x_91); -x_77 = x_86; -x_78 = x_88; +x_77 = x_88; +x_78 = x_86; x_79 = x_87; x_80 = x_92; goto block_85; @@ -28990,7 +28990,7 @@ goto block_208; { 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; x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_173); +lean_ctor_set(x_176, 0, x_172); lean_ctor_set(x_176, 1, x_175); x_177 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__8; x_178 = lean_alloc_ctor(3, 1, 0); @@ -29011,13 +29011,13 @@ lean_dec(x_171); x_185 = l_List_appendTR___redArg(x_182, x_184); x_186 = l_Lean_Json_mkObj(x_185); x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_172); +lean_ctor_set(x_187, 0, x_174); lean_ctor_set(x_187, 1, x_186); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_187); lean_ctor_set(x_188, 1, x_180); x_189 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_189, 0, x_174); +lean_ctor_set(x_189, 0, x_173); lean_ctor_set(x_189, 1, x_188); x_109 = x_189; goto block_118; @@ -29035,9 +29035,9 @@ case 0: { lean_object* x_196; x_196 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__15; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_196; goto block_190; } @@ -29045,9 +29045,9 @@ case 1: { lean_object* x_197; x_197 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__19; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_197; goto block_190; } @@ -29055,9 +29055,9 @@ case 2: { lean_object* x_198; x_198 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__23; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_198; goto block_190; } @@ -29065,9 +29065,9 @@ case 3: { lean_object* x_199; x_199 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__27; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_199; goto block_190; } @@ -29075,9 +29075,9 @@ case 4: { lean_object* x_200; x_200 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__31; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_200; goto block_190; } @@ -29085,9 +29085,9 @@ case 5: { lean_object* x_201; x_201 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__35; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_201; goto block_190; } @@ -29095,9 +29095,9 @@ case 6: { lean_object* x_202; x_202 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__39; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_202; goto block_190; } @@ -29105,9 +29105,9 @@ case 7: { lean_object* x_203; x_203 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__43; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_203; goto block_190; } @@ -29115,9 +29115,9 @@ case 8: { lean_object* x_204; x_204 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__47; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_204; goto block_190; } @@ -29125,9 +29125,9 @@ case 9: { lean_object* x_205; x_205 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__51; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_205; goto block_190; } @@ -29135,9 +29135,9 @@ case 10: { lean_object* x_206; x_206 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__55; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_206; goto block_190; } @@ -29145,9 +29145,9 @@ goto block_190; { lean_object* x_207; x_207 = l_Lean_Server_FileWorker_OutputMessage_ofMsg___closed__59; -x_172 = x_194; -x_173 = x_195; -x_174 = x_193; +x_172 = x_195; +x_173 = x_193; +x_174 = x_194; x_175 = x_207; goto block_190; } diff --git a/stage0/stdlib/Lean/Server/Test/Runner.c b/stage0/stdlib/Lean/Server/Test/Runner.c index 8fec93a54f30..93df8f76e747 100644 --- a/stage0/stdlib/Lean/Server/Test/Runner.c +++ b/stage0/stdlib/Lean/Server/Test/Runner.c @@ -20485,8 +20485,8 @@ x_62 = 97; x_63 = lean_uint32_dec_le(x_62, x_59); if (x_63 == 0) { -lean_dec_ref(x_61); -x_55 = x_60; +lean_dec_ref(x_60); +x_55 = x_61; goto block_58; } else @@ -20496,15 +20496,15 @@ x_64 = 122; x_65 = lean_uint32_dec_le(x_59, x_64); if (x_65 == 0) { -lean_dec_ref(x_61); -x_55 = x_60; +lean_dec_ref(x_60); +x_55 = x_61; goto block_58; } else { -lean_dec_ref(x_60); +lean_dec_ref(x_61); lean_dec(x_9); -x_3 = x_61; +x_3 = x_60; x_4 = x_59; goto block_7; } @@ -20551,8 +20551,8 @@ x_78 = lean_uint32_dec_le(x_77, x_74); if (x_78 == 0) { x_59 = x_74; -x_60 = x_68; -x_61 = x_76; +x_60 = x_76; +x_61 = x_68; goto block_66; } else @@ -20563,8 +20563,8 @@ x_80 = lean_uint32_dec_le(x_74, x_79); if (x_80 == 0) { x_59 = x_74; -x_60 = x_68; -x_61 = x_76; +x_60 = x_76; +x_61 = x_68; goto block_66; } else @@ -20607,7 +20607,7 @@ goto block_81; LEAN_EXPORT lean_object* l_Lean_Server_Test_Runner_word(lean_object* x_1) { _start: { -lean_object* x_2; uint32_t x_3; lean_object* x_8; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_56; lean_object* x_60; uint32_t x_64; lean_object* x_65; lean_object* x_66; 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_92; uint8_t x_93; +lean_object* x_2; uint32_t x_3; lean_object* x_8; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_56; lean_object* x_60; lean_object* x_64; uint32_t x_65; lean_object* x_66; 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_92; uint8_t x_93; x_72 = lean_ctor_get(x_1, 0); lean_inc(x_72); x_73 = lean_ctor_get(x_1, 1); @@ -20938,29 +20938,29 @@ goto block_55; { uint32_t x_67; uint8_t x_68; x_67 = 97; -x_68 = lean_uint32_dec_le(x_67, x_64); +x_68 = lean_uint32_dec_le(x_67, x_65); if (x_68 == 0) { -lean_dec_ref(x_66); -x_56 = x_65; +lean_dec_ref(x_64); +x_56 = x_66; goto block_59; } else { uint32_t x_69; uint8_t x_70; x_69 = 122; -x_70 = lean_uint32_dec_le(x_64, x_69); +x_70 = lean_uint32_dec_le(x_65, x_69); if (x_70 == 0) { -lean_dec_ref(x_66); -x_56 = x_65; +lean_dec_ref(x_64); +x_56 = x_66; goto block_59; } else { -lean_dec_ref(x_65); -x_2 = x_66; -x_3 = x_64; +lean_dec_ref(x_66); +x_2 = x_64; +x_3 = x_65; goto block_7; } } @@ -21008,9 +21008,9 @@ x_85 = 65; x_86 = lean_uint32_dec_le(x_85, x_82); if (x_86 == 0) { -x_64 = x_82; -x_65 = x_74; -x_66 = x_84; +x_64 = x_84; +x_65 = x_82; +x_66 = x_74; goto block_71; } else @@ -21020,9 +21020,9 @@ x_87 = 90; x_88 = lean_uint32_dec_le(x_82, x_87); if (x_88 == 0) { -x_64 = x_82; -x_65 = x_74; -x_66 = x_84; +x_64 = x_84; +x_65 = x_82; +x_66 = x_74; goto block_71; } else @@ -23049,9 +23049,9 @@ goto block_190; block_182: { lean_object* x_179; lean_object* x_180; lean_object* x_181; -x_179 = lean_nat_add(x_177, x_178); +x_179 = lean_nat_add(x_176, x_178); lean_dec(x_178); -lean_dec(x_177); +lean_dec(x_176); if (lean_is_scalar(x_172)) { x_180 = lean_alloc_ctor(0, 5, 0); } else { @@ -23070,7 +23070,7 @@ if (lean_is_scalar(x_162)) { lean_ctor_set(x_181, 0, x_175); lean_ctor_set(x_181, 1, x_165); lean_ctor_set(x_181, 2, x_166); -lean_ctor_set(x_181, 3, x_176); +lean_ctor_set(x_181, 3, x_177); lean_ctor_set(x_181, 4, x_180); return x_181; } @@ -23096,8 +23096,8 @@ if (lean_obj_tag(x_168) == 0) lean_object* x_188; x_188 = lean_ctor_get(x_168, 0); lean_inc(x_188); -x_176 = x_186; -x_177 = x_187; +x_176 = x_187; +x_177 = x_186; x_178 = x_188; goto block_182; } @@ -23105,8 +23105,8 @@ else { lean_object* x_189; x_189 = lean_unsigned_to_nat(0u); -x_176 = x_186; -x_177 = x_187; +x_176 = x_187; +x_177 = x_186; x_178 = x_189; goto block_182; } @@ -28467,7 +28467,7 @@ goto block_138; { 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; x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 0, x_95); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_100 = lean_alloc_ctor(3, 1, 0); @@ -28488,7 +28488,7 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_95); +lean_ctor_set(x_109, 0, x_96); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); @@ -28529,8 +28529,8 @@ case 0: lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_126; goto block_120; } @@ -28539,8 +28539,8 @@ case 1: lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_127; goto block_120; } @@ -28549,8 +28549,8 @@ case 2: lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_128; goto block_120; } @@ -28559,8 +28559,8 @@ case 3: lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_129; goto block_120; } @@ -28569,8 +28569,8 @@ case 4: lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_130; goto block_120; } @@ -28579,8 +28579,8 @@ case 5: lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_131; goto block_120; } @@ -28589,8 +28589,8 @@ case 6: lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_132; goto block_120; } @@ -28599,8 +28599,8 @@ case 7: lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_133; goto block_120; } @@ -28609,8 +28609,8 @@ case 8: lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_134; goto block_120; } @@ -28619,8 +28619,8 @@ case 9: lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_135; goto block_120; } @@ -28629,8 +28629,8 @@ case 10: lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_136; goto block_120; } @@ -28639,8 +28639,8 @@ goto block_120; lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; x_94 = x_123; -x_95 = x_124; -x_96 = x_125; +x_95 = x_125; +x_96 = x_124; x_97 = x_137; goto block_120; } @@ -31429,7 +31429,7 @@ goto block_116; { 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; x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 0, x_73); lean_ctor_set(x_76, 1, x_75); x_77 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_78 = lean_alloc_ctor(3, 1, 0); @@ -31450,13 +31450,13 @@ lean_dec(x_69); x_85 = l_List_appendTR___redArg(x_82, x_84); x_86 = l_Lean_Json_mkObj(x_85); x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_72); +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_87); lean_ctor_set(x_88, 1, x_80); x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_73); +lean_ctor_set(x_89, 0, x_72); lean_ctor_set(x_89, 1, x_88); x_90 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_90, 0, x_71); @@ -31490,9 +31490,9 @@ case 0: { lean_object* x_104; x_104 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_104; goto block_98; } @@ -31500,9 +31500,9 @@ case 1: { lean_object* x_105; x_105 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_105; goto block_98; } @@ -31510,9 +31510,9 @@ case 2: { lean_object* x_106; x_106 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_106; goto block_98; } @@ -31520,9 +31520,9 @@ case 3: { lean_object* x_107; x_107 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_107; goto block_98; } @@ -31530,9 +31530,9 @@ case 4: { lean_object* x_108; x_108 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_108; goto block_98; } @@ -31540,9 +31540,9 @@ case 5: { lean_object* x_109; x_109 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_109; goto block_98; } @@ -31550,9 +31550,9 @@ case 6: { lean_object* x_110; x_110 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_110; goto block_98; } @@ -31560,9 +31560,9 @@ case 7: { lean_object* x_111; x_111 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_111; goto block_98; } @@ -31570,9 +31570,9 @@ case 8: { lean_object* x_112; x_112 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_112; goto block_98; } @@ -31580,9 +31580,9 @@ case 9: { lean_object* x_113; x_113 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_113; goto block_98; } @@ -31590,9 +31590,9 @@ case 10: { lean_object* x_114; x_114 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_114; goto block_98; } @@ -31600,9 +31600,9 @@ goto block_98; { lean_object* x_115; x_115 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_72 = x_102; -x_73 = x_101; -x_74 = x_103; +x_72 = x_101; +x_73 = x_103; +x_74 = x_102; x_75 = x_115; goto block_98; } @@ -32523,7 +32523,7 @@ goto block_138; { 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; x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 0, x_94); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_100 = lean_alloc_ctor(3, 1, 0); @@ -32550,7 +32550,7 @@ x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_94); +lean_ctor_set(x_111, 0, x_96); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -32584,9 +32584,9 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_126; goto block_120; } @@ -32594,9 +32594,9 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_127; goto block_120; } @@ -32604,9 +32604,9 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_128; goto block_120; } @@ -32614,9 +32614,9 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_129; goto block_120; } @@ -32624,9 +32624,9 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_130; goto block_120; } @@ -32634,9 +32634,9 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_131; goto block_120; } @@ -32644,9 +32644,9 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_132; goto block_120; } @@ -32654,9 +32654,9 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_133; goto block_120; } @@ -32664,9 +32664,9 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_134; goto block_120; } @@ -32674,9 +32674,9 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_135; goto block_120; } @@ -32684,9 +32684,9 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_136; goto block_120; } @@ -32694,9 +32694,9 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_123; +x_94 = x_125; x_95 = x_124; -x_96 = x_125; +x_96 = x_123; x_97 = x_137; goto block_120; } @@ -35996,7 +35996,7 @@ goto block_138; { 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; x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 0, x_96); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_100 = lean_alloc_ctor(3, 1, 0); @@ -36017,13 +36017,13 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_96); +lean_ctor_set(x_109, 0, x_94); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_94); +lean_ctor_set(x_111, 0, x_95); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -36057,9 +36057,9 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_126; goto block_120; } @@ -36067,9 +36067,9 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_127; goto block_120; } @@ -36077,9 +36077,9 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_128; goto block_120; } @@ -36087,9 +36087,9 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_129; goto block_120; } @@ -36097,9 +36097,9 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_130; goto block_120; } @@ -36107,9 +36107,9 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_131; goto block_120; } @@ -36117,9 +36117,9 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_132; goto block_120; } @@ -36127,9 +36127,9 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_133; goto block_120; } @@ -36137,9 +36137,9 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_134; goto block_120; } @@ -36147,9 +36147,9 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_135; goto block_120; } @@ -36157,9 +36157,9 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_136; goto block_120; } @@ -36167,9 +36167,9 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_124; +x_95 = x_123; +x_96 = x_125; x_97 = x_137; goto block_120; } @@ -38591,13 +38591,13 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_94); +lean_ctor_set(x_109, 0, x_95); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_95); +lean_ctor_set(x_111, 0, x_94); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -38631,8 +38631,8 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_126; goto block_120; @@ -38641,8 +38641,8 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_127; goto block_120; @@ -38651,8 +38651,8 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_128; goto block_120; @@ -38661,8 +38661,8 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_129; goto block_120; @@ -38671,8 +38671,8 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_130; goto block_120; @@ -38681,8 +38681,8 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_131; goto block_120; @@ -38691,8 +38691,8 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_132; goto block_120; @@ -38701,8 +38701,8 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_133; goto block_120; @@ -38711,8 +38711,8 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_134; goto block_120; @@ -38721,8 +38721,8 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_135; goto block_120; @@ -38731,8 +38731,8 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_136; goto block_120; @@ -38741,8 +38741,8 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_137; goto block_120; @@ -41942,13 +41942,13 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_94); +lean_ctor_set(x_109, 0, x_96); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_96); +lean_ctor_set(x_111, 0, x_94); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -41982,9 +41982,9 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_126; goto block_120; } @@ -41992,9 +41992,9 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_127; goto block_120; } @@ -42002,9 +42002,9 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_128; goto block_120; } @@ -42012,9 +42012,9 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_129; goto block_120; } @@ -42022,9 +42022,9 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_130; goto block_120; } @@ -42032,9 +42032,9 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_131; goto block_120; } @@ -42042,9 +42042,9 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_132; goto block_120; } @@ -42052,9 +42052,9 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_133; goto block_120; } @@ -42062,9 +42062,9 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_134; goto block_120; } @@ -42072,9 +42072,9 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_135; goto block_120; } @@ -42082,9 +42082,9 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_136; goto block_120; } @@ -42092,9 +42092,9 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_124; +x_94 = x_123; x_95 = x_125; -x_96 = x_123; +x_96 = x_124; x_97 = x_137; goto block_120; } @@ -45498,7 +45498,7 @@ goto block_138; { 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; x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 0, x_94); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_100 = lean_alloc_ctor(3, 1, 0); @@ -45519,7 +45519,7 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_94); +lean_ctor_set(x_109, 0, x_96); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); @@ -45559,9 +45559,9 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_126; goto block_120; } @@ -45569,9 +45569,9 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_127; goto block_120; } @@ -45579,9 +45579,9 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_128; goto block_120; } @@ -45589,9 +45589,9 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_129; goto block_120; } @@ -45599,9 +45599,9 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_130; goto block_120; } @@ -45609,9 +45609,9 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_131; goto block_120; } @@ -45619,9 +45619,9 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_132; goto block_120; } @@ -45629,9 +45629,9 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_133; goto block_120; } @@ -45639,9 +45639,9 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_134; goto block_120; } @@ -45649,9 +45649,9 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_135; goto block_120; } @@ -45659,9 +45659,9 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_136; goto block_120; } @@ -45669,9 +45669,9 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_124; +x_94 = x_125; x_95 = x_123; -x_96 = x_125; +x_96 = x_124; x_97 = x_137; goto block_120; } @@ -47246,7 +47246,7 @@ goto block_138; { 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; x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 0, x_94); lean_ctor_set(x_98, 1, x_97); x_99 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__11; x_100 = lean_alloc_ctor(3, 1, 0); @@ -47267,13 +47267,13 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_96); +lean_ctor_set(x_109, 0, x_95); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_94); +lean_ctor_set(x_111, 0, x_96); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -47307,9 +47307,9 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_126; goto block_120; } @@ -47317,9 +47317,9 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_127; goto block_120; } @@ -47327,9 +47327,9 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_128; goto block_120; } @@ -47337,9 +47337,9 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_129; goto block_120; } @@ -47347,9 +47347,9 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_130; goto block_120; } @@ -47357,9 +47357,9 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_131; goto block_120; } @@ -47367,9 +47367,9 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_132; goto block_120; } @@ -47377,9 +47377,9 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_133; goto block_120; } @@ -47387,9 +47387,9 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_134; goto block_120; } @@ -47397,9 +47397,9 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_135; goto block_120; } @@ -47407,9 +47407,9 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_136; goto block_120; } @@ -47417,9 +47417,9 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_123; -x_95 = x_125; -x_96 = x_124; +x_94 = x_125; +x_95 = x_124; +x_96 = x_123; x_97 = x_137; goto block_120; } @@ -53895,108 +53895,108 @@ x_12 = lean_ctor_get(x_4, 5); lean_dec(x_12); x_13 = lean_ctor_get(x_4, 4); lean_dec(x_13); -lean_inc_ref(x_7); +lean_inc_ref(x_8); lean_ctor_set(x_4, 6, x_9); -lean_ctor_set(x_4, 5, x_7); -lean_ctor_set(x_4, 4, x_8); +lean_ctor_set(x_4, 5, x_8); +lean_ctor_set(x_4, 4, x_7); x_14 = l_Lean_Server_Test_Runner_processEdit___closed__6; -x_15 = lean_string_dec_eq(x_7, x_14); +x_15 = lean_string_dec_eq(x_8, x_14); if (x_15 == 0) { lean_object* x_16; uint8_t x_17; x_16 = l_Lean_Server_Test_Runner_processEdit___closed__7; -x_17 = lean_string_dec_eq(x_7, x_16); +x_17 = lean_string_dec_eq(x_8, x_16); if (x_17 == 0) { lean_object* x_18; uint8_t x_19; x_18 = l_Lean_Server_Test_Runner_processEdit___closed__8; -x_19 = lean_string_dec_eq(x_7, x_18); +x_19 = lean_string_dec_eq(x_8, x_18); if (x_19 == 0) { lean_object* x_20; uint8_t x_21; x_20 = l_Lean_Server_Test_Runner_processDirective___closed__0; -x_21 = lean_string_dec_eq(x_7, x_20); +x_21 = lean_string_dec_eq(x_8, x_20); if (x_21 == 0) { lean_object* x_22; uint8_t x_23; x_22 = l_Lean_Server_Test_Runner_processDirective___closed__1; -x_23 = lean_string_dec_eq(x_7, x_22); +x_23 = lean_string_dec_eq(x_8, x_22); if (x_23 == 0) { lean_object* x_24; uint8_t x_25; x_24 = l_Lean_Server_Test_Runner_processDirective___closed__2; -x_25 = lean_string_dec_eq(x_7, x_24); +x_25 = lean_string_dec_eq(x_8, x_24); if (x_25 == 0) { lean_object* x_26; uint8_t x_27; x_26 = l_Lean_Server_Test_Runner_processDirective___closed__3; -x_27 = lean_string_dec_eq(x_7, x_26); +x_27 = lean_string_dec_eq(x_8, x_26); if (x_27 == 0) { lean_object* x_28; uint8_t x_29; x_28 = l_Lean_Server_Test_Runner_processDirective___closed__4; -x_29 = lean_string_dec_eq(x_7, x_28); +x_29 = lean_string_dec_eq(x_8, x_28); if (x_29 == 0) { lean_object* x_30; uint8_t x_31; x_30 = l_Lean_Server_Test_Runner_processDirective___closed__5; -x_31 = lean_string_dec_eq(x_7, x_30); +x_31 = lean_string_dec_eq(x_8, x_30); if (x_31 == 0) { lean_object* x_32; uint8_t x_33; x_32 = l_Lean_Server_Test_Runner_Client_instFromJsonInteractiveGoals_fromJson___closed__0; -x_33 = lean_string_dec_eq(x_7, x_32); +x_33 = lean_string_dec_eq(x_8, x_32); if (x_33 == 0) { lean_object* x_34; uint8_t x_35; x_34 = l_Lean_Server_Test_Runner_processDirective___closed__6; -x_35 = lean_string_dec_eq(x_7, x_34); +x_35 = lean_string_dec_eq(x_8, x_34); if (x_35 == 0) { lean_object* x_36; uint8_t x_37; x_36 = l_Lean_Server_Test_Runner_instFromJsonGetWidgetsResponse_fromJson___closed__0; -x_37 = lean_string_dec_eq(x_7, x_36); +x_37 = lean_string_dec_eq(x_8, x_36); if (x_37 == 0) { lean_object* x_38; uint8_t x_39; x_38 = l_Lean_Server_Test_Runner_processDirective___closed__7; -x_39 = lean_string_dec_eq(x_7, x_38); +x_39 = lean_string_dec_eq(x_8, x_38); if (x_39 == 0) { lean_object* x_40; uint8_t x_41; x_40 = l_Lean_Server_Test_Runner_processDirective___closed__8; -x_41 = lean_string_dec_eq(x_7, x_40); +x_41 = lean_string_dec_eq(x_8, x_40); if (x_41 == 0) { lean_object* x_42; uint8_t x_43; x_42 = l_Lean_Server_Test_Runner_processDirective___closed__9; -x_43 = lean_string_dec_eq(x_7, x_42); +x_43 = lean_string_dec_eq(x_8, x_42); if (x_43 == 0) { lean_object* x_44; uint8_t x_45; x_44 = l_Lean_Server_Test_Runner_processDirective___closed__10; -x_45 = lean_string_dec_eq(x_7, x_44); +x_45 = lean_string_dec_eq(x_8, x_44); if (x_45 == 0) { lean_object* x_46; uint8_t x_47; x_46 = l_Lean_Server_Test_Runner_processDirective___closed__11; -x_47 = lean_string_dec_eq(x_7, x_46); +x_47 = lean_string_dec_eq(x_8, x_46); if (x_47 == 0) { lean_object* x_48; uint8_t x_49; x_48 = l_Lean_Server_Test_Runner_processDirective___closed__12; -x_49 = lean_string_dec_eq(x_7, x_48); +x_49 = lean_string_dec_eq(x_8, x_48); if (x_49 == 0) { lean_object* x_50; uint8_t x_51; x_50 = l_Lean_Server_Test_Runner_processDirective___closed__13; -x_51 = lean_string_dec_eq(x_7, x_50); +x_51 = lean_string_dec_eq(x_8, x_50); if (x_51 == 0) { lean_object* x_52; uint8_t x_53; x_52 = l_Lean_Server_Test_Runner_processDirective___closed__14; -x_53 = lean_string_dec_eq(x_7, x_52); -lean_dec_ref(x_7); +x_53 = lean_string_dec_eq(x_8, x_52); +lean_dec_ref(x_8); if (x_53 == 0) { lean_object* x_54; @@ -54013,7 +54013,7 @@ return x_55; else { lean_object* x_56; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_56 = l_Lean_Server_Test_Runner_processModuleHierarchyImportedBy(x_4, x_5); return x_56; } @@ -54021,7 +54021,7 @@ return x_56; else { lean_object* x_57; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_57 = l_Lean_Server_Test_Runner_processModuleHierarchyImports(x_4, x_5); return x_57; } @@ -54029,7 +54029,7 @@ return x_57; else { lean_object* x_58; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_58 = l_Lean_Server_Test_Runner_processSymbols(x_4, x_5); return x_58; } @@ -54037,7 +54037,7 @@ return x_58; else { lean_object* x_59; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_59 = l_Lean_Server_Test_Runner_processReferences(x_4, x_5); return x_59; } @@ -54045,7 +54045,7 @@ return x_59; else { lean_object* x_60; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_60 = l_Lean_Server_Test_Runner_processOutgoingCallHierarchy(x_4, x_5); return x_60; } @@ -54053,7 +54053,7 @@ return x_60; else { lean_object* x_61; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_61 = l_Lean_Server_Test_Runner_processIncomingCallHierarchy(x_4, x_5); return x_61; } @@ -54061,7 +54061,7 @@ return x_61; else { lean_object* x_62; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_62 = l_Lean_Server_Test_Runner_processCompletion(x_4, x_5); return x_62; } @@ -54069,7 +54069,7 @@ return x_62; else { lean_object* x_63; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_63 = l_Lean_Server_Test_Runner_processWidgets(x_4, x_5); return x_63; } @@ -54077,7 +54077,7 @@ return x_63; else { lean_object* x_64; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_64 = l_Lean_Server_Test_Runner_processTermGoal(x_4, x_5); return x_64; } @@ -54085,7 +54085,7 @@ return x_64; else { lean_object* x_65; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_65 = l_Lean_Server_Test_Runner_processGoals(x_4, x_5); return x_65; } @@ -54093,7 +54093,7 @@ return x_65; else { lean_object* x_66; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_66 = l_Lean_Server_Test_Runner_processInteractiveDiagnostics(x_4, x_5); return x_66; } @@ -54101,7 +54101,7 @@ return x_66; else { lean_object* x_67; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_67 = l_Lean_Server_Test_Runner_processCodeAction(x_4, x_5); return x_67; } @@ -54109,7 +54109,7 @@ return x_67; else { lean_object* x_68; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_68 = l_Lean_Server_Test_Runner_processWaitFor(x_4, x_5); return x_68; } @@ -54117,7 +54117,7 @@ return x_68; else { lean_object* x_69; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_69 = l_Lean_Server_Test_Runner_processSync(x_4, x_5); return x_69; } @@ -54125,7 +54125,7 @@ return x_69; else { lean_object* x_70; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_70 = l_Lean_Server_Test_Runner_processWaitForILeans(x_4, x_5); return x_70; } @@ -54133,7 +54133,7 @@ return x_70; else { lean_object* x_71; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_71 = l_Lean_Server_Test_Runner_processCollectDiagnostics(x_4, x_5); return x_71; } @@ -54141,7 +54141,7 @@ return x_71; else { lean_object* x_72; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_72 = l_Lean_Server_Test_Runner_processEdit(x_4, x_5); return x_72; } @@ -54149,7 +54149,7 @@ return x_72; else { lean_object* x_73; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_73 = l_Lean_Server_Test_Runner_processEdit(x_4, x_5); return x_73; } @@ -54157,7 +54157,7 @@ return x_73; else { lean_object* x_74; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_74 = l_Lean_Server_Test_Runner_processEdit(x_4, x_5); return x_74; } @@ -54179,116 +54179,116 @@ lean_inc(x_78); lean_inc(x_77); lean_inc(x_75); lean_dec(x_4); -lean_inc_ref(x_7); +lean_inc_ref(x_8); x_82 = lean_alloc_ctor(0, 9, 1); lean_ctor_set(x_82, 0, x_75); lean_ctor_set(x_82, 1, x_77); lean_ctor_set(x_82, 2, x_78); lean_ctor_set(x_82, 3, x_79); -lean_ctor_set(x_82, 4, x_8); -lean_ctor_set(x_82, 5, x_7); +lean_ctor_set(x_82, 4, x_7); +lean_ctor_set(x_82, 5, x_8); lean_ctor_set(x_82, 6, x_9); lean_ctor_set(x_82, 7, x_80); lean_ctor_set(x_82, 8, x_81); lean_ctor_set_uint8(x_82, sizeof(void*)*9, x_76); x_83 = l_Lean_Server_Test_Runner_processEdit___closed__6; -x_84 = lean_string_dec_eq(x_7, x_83); +x_84 = lean_string_dec_eq(x_8, x_83); if (x_84 == 0) { lean_object* x_85; uint8_t x_86; x_85 = l_Lean_Server_Test_Runner_processEdit___closed__7; -x_86 = lean_string_dec_eq(x_7, x_85); +x_86 = lean_string_dec_eq(x_8, x_85); if (x_86 == 0) { lean_object* x_87; uint8_t x_88; x_87 = l_Lean_Server_Test_Runner_processEdit___closed__8; -x_88 = lean_string_dec_eq(x_7, x_87); +x_88 = lean_string_dec_eq(x_8, x_87); if (x_88 == 0) { lean_object* x_89; uint8_t x_90; x_89 = l_Lean_Server_Test_Runner_processDirective___closed__0; -x_90 = lean_string_dec_eq(x_7, x_89); +x_90 = lean_string_dec_eq(x_8, x_89); if (x_90 == 0) { lean_object* x_91; uint8_t x_92; x_91 = l_Lean_Server_Test_Runner_processDirective___closed__1; -x_92 = lean_string_dec_eq(x_7, x_91); +x_92 = lean_string_dec_eq(x_8, x_91); if (x_92 == 0) { lean_object* x_93; uint8_t x_94; x_93 = l_Lean_Server_Test_Runner_processDirective___closed__2; -x_94 = lean_string_dec_eq(x_7, x_93); +x_94 = lean_string_dec_eq(x_8, x_93); if (x_94 == 0) { lean_object* x_95; uint8_t x_96; x_95 = l_Lean_Server_Test_Runner_processDirective___closed__3; -x_96 = lean_string_dec_eq(x_7, x_95); +x_96 = lean_string_dec_eq(x_8, x_95); if (x_96 == 0) { lean_object* x_97; uint8_t x_98; x_97 = l_Lean_Server_Test_Runner_processDirective___closed__4; -x_98 = lean_string_dec_eq(x_7, x_97); +x_98 = lean_string_dec_eq(x_8, x_97); if (x_98 == 0) { lean_object* x_99; uint8_t x_100; x_99 = l_Lean_Server_Test_Runner_processDirective___closed__5; -x_100 = lean_string_dec_eq(x_7, x_99); +x_100 = lean_string_dec_eq(x_8, x_99); if (x_100 == 0) { lean_object* x_101; uint8_t x_102; x_101 = l_Lean_Server_Test_Runner_Client_instFromJsonInteractiveGoals_fromJson___closed__0; -x_102 = lean_string_dec_eq(x_7, x_101); +x_102 = lean_string_dec_eq(x_8, x_101); if (x_102 == 0) { lean_object* x_103; uint8_t x_104; x_103 = l_Lean_Server_Test_Runner_processDirective___closed__6; -x_104 = lean_string_dec_eq(x_7, x_103); +x_104 = lean_string_dec_eq(x_8, x_103); if (x_104 == 0) { lean_object* x_105; uint8_t x_106; x_105 = l_Lean_Server_Test_Runner_instFromJsonGetWidgetsResponse_fromJson___closed__0; -x_106 = lean_string_dec_eq(x_7, x_105); +x_106 = lean_string_dec_eq(x_8, x_105); if (x_106 == 0) { lean_object* x_107; uint8_t x_108; x_107 = l_Lean_Server_Test_Runner_processDirective___closed__7; -x_108 = lean_string_dec_eq(x_7, x_107); +x_108 = lean_string_dec_eq(x_8, x_107); if (x_108 == 0) { lean_object* x_109; uint8_t x_110; x_109 = l_Lean_Server_Test_Runner_processDirective___closed__8; -x_110 = lean_string_dec_eq(x_7, x_109); +x_110 = lean_string_dec_eq(x_8, x_109); if (x_110 == 0) { lean_object* x_111; uint8_t x_112; x_111 = l_Lean_Server_Test_Runner_processDirective___closed__9; -x_112 = lean_string_dec_eq(x_7, x_111); +x_112 = lean_string_dec_eq(x_8, x_111); if (x_112 == 0) { lean_object* x_113; uint8_t x_114; x_113 = l_Lean_Server_Test_Runner_processDirective___closed__10; -x_114 = lean_string_dec_eq(x_7, x_113); +x_114 = lean_string_dec_eq(x_8, x_113); if (x_114 == 0) { lean_object* x_115; uint8_t x_116; x_115 = l_Lean_Server_Test_Runner_processDirective___closed__11; -x_116 = lean_string_dec_eq(x_7, x_115); +x_116 = lean_string_dec_eq(x_8, x_115); if (x_116 == 0) { lean_object* x_117; uint8_t x_118; x_117 = l_Lean_Server_Test_Runner_processDirective___closed__12; -x_118 = lean_string_dec_eq(x_7, x_117); +x_118 = lean_string_dec_eq(x_8, x_117); if (x_118 == 0) { lean_object* x_119; uint8_t x_120; x_119 = l_Lean_Server_Test_Runner_processDirective___closed__13; -x_120 = lean_string_dec_eq(x_7, x_119); +x_120 = lean_string_dec_eq(x_8, x_119); if (x_120 == 0) { lean_object* x_121; uint8_t x_122; x_121 = l_Lean_Server_Test_Runner_processDirective___closed__14; -x_122 = lean_string_dec_eq(x_7, x_121); -lean_dec_ref(x_7); +x_122 = lean_string_dec_eq(x_8, x_121); +lean_dec_ref(x_8); if (x_122 == 0) { lean_object* x_123; @@ -54305,7 +54305,7 @@ return x_124; else { lean_object* x_125; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_125 = l_Lean_Server_Test_Runner_processModuleHierarchyImportedBy(x_82, x_5); return x_125; } @@ -54313,7 +54313,7 @@ return x_125; else { lean_object* x_126; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_126 = l_Lean_Server_Test_Runner_processModuleHierarchyImports(x_82, x_5); return x_126; } @@ -54321,7 +54321,7 @@ return x_126; else { lean_object* x_127; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_127 = l_Lean_Server_Test_Runner_processSymbols(x_82, x_5); return x_127; } @@ -54329,7 +54329,7 @@ return x_127; else { lean_object* x_128; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_128 = l_Lean_Server_Test_Runner_processReferences(x_82, x_5); return x_128; } @@ -54337,7 +54337,7 @@ return x_128; else { lean_object* x_129; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_129 = l_Lean_Server_Test_Runner_processOutgoingCallHierarchy(x_82, x_5); return x_129; } @@ -54345,7 +54345,7 @@ return x_129; else { lean_object* x_130; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_130 = l_Lean_Server_Test_Runner_processIncomingCallHierarchy(x_82, x_5); return x_130; } @@ -54353,7 +54353,7 @@ return x_130; else { lean_object* x_131; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_131 = l_Lean_Server_Test_Runner_processCompletion(x_82, x_5); return x_131; } @@ -54361,7 +54361,7 @@ return x_131; else { lean_object* x_132; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_132 = l_Lean_Server_Test_Runner_processWidgets(x_82, x_5); return x_132; } @@ -54369,7 +54369,7 @@ return x_132; else { lean_object* x_133; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_133 = l_Lean_Server_Test_Runner_processTermGoal(x_82, x_5); return x_133; } @@ -54377,7 +54377,7 @@ return x_133; else { lean_object* x_134; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_134 = l_Lean_Server_Test_Runner_processGoals(x_82, x_5); return x_134; } @@ -54385,7 +54385,7 @@ return x_134; else { lean_object* x_135; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_135 = l_Lean_Server_Test_Runner_processInteractiveDiagnostics(x_82, x_5); return x_135; } @@ -54393,7 +54393,7 @@ return x_135; else { lean_object* x_136; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_136 = l_Lean_Server_Test_Runner_processCodeAction(x_82, x_5); return x_136; } @@ -54401,7 +54401,7 @@ return x_136; else { lean_object* x_137; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_137 = l_Lean_Server_Test_Runner_processWaitFor(x_82, x_5); return x_137; } @@ -54409,7 +54409,7 @@ return x_137; else { lean_object* x_138; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_138 = l_Lean_Server_Test_Runner_processSync(x_82, x_5); return x_138; } @@ -54417,7 +54417,7 @@ return x_138; else { lean_object* x_139; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_139 = l_Lean_Server_Test_Runner_processWaitForILeans(x_82, x_5); return x_139; } @@ -54425,7 +54425,7 @@ return x_139; else { lean_object* x_140; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_140 = l_Lean_Server_Test_Runner_processCollectDiagnostics(x_82, x_5); return x_140; } @@ -54433,7 +54433,7 @@ return x_140; else { lean_object* x_141; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_141 = l_Lean_Server_Test_Runner_processEdit(x_82, x_5); return x_141; } @@ -54441,7 +54441,7 @@ return x_141; else { lean_object* x_142; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_142 = l_Lean_Server_Test_Runner_processEdit(x_82, x_5); return x_142; } @@ -54449,7 +54449,7 @@ return x_142; else { lean_object* x_143; -lean_dec_ref(x_7); +lean_dec_ref(x_8); x_143 = l_Lean_Server_Test_Runner_processEdit(x_82, x_5); return x_143; } @@ -54514,8 +54514,8 @@ x_172 = lean_string_utf8_extract(x_169, x_170, x_171); lean_dec(x_171); lean_dec(x_170); lean_dec_ref(x_169); -x_7 = x_158; -x_8 = x_162; +x_7 = x_162; +x_8 = x_158; x_9 = x_172; goto block_144; } @@ -54527,8 +54527,8 @@ lean_dec(x_151); lean_dec(x_149); lean_dec_ref(x_2); x_173 = l_Lean_Server_Test_Runner_processDirective___closed__17; -x_7 = x_158; -x_8 = x_162; +x_7 = x_162; +x_8 = x_158; x_9 = x_173; goto block_144; } @@ -54583,8 +54583,8 @@ x_192 = lean_string_utf8_extract(x_189, x_190, x_191); lean_dec(x_191); lean_dec(x_190); lean_dec_ref(x_189); -x_7 = x_177; -x_8 = x_181; +x_7 = x_181; +x_8 = x_177; x_9 = x_192; goto block_144; } @@ -54595,8 +54595,8 @@ lean_dec(x_151); lean_dec(x_149); lean_dec_ref(x_2); x_193 = l_Lean_Server_Test_Runner_processDirective___closed__17; -x_7 = x_177; -x_8 = x_181; +x_7 = x_181; +x_8 = x_177; x_9 = x_193; goto block_144; } @@ -57706,13 +57706,13 @@ lean_dec(x_91); x_107 = l_List_appendTR___redArg(x_104, x_106); x_108 = l_Lean_Json_mkObj(x_107); x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_94); +lean_ctor_set(x_109, 0, x_95); lean_ctor_set(x_109, 1, x_108); x_110 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_110, 0, x_109); lean_ctor_set(x_110, 1, x_102); x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_95); +lean_ctor_set(x_111, 0, x_94); lean_ctor_set(x_111, 1, x_110); x_112 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_112, 0, x_93); @@ -57746,8 +57746,8 @@ case 0: { lean_object* x_126; x_126 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__18; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_126; goto block_120; @@ -57756,8 +57756,8 @@ case 1: { lean_object* x_127; x_127 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__22; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_127; goto block_120; @@ -57766,8 +57766,8 @@ case 2: { lean_object* x_128; x_128 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__26; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_128; goto block_120; @@ -57776,8 +57776,8 @@ case 3: { lean_object* x_129; x_129 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__30; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_129; goto block_120; @@ -57786,8 +57786,8 @@ case 4: { lean_object* x_130; x_130 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__34; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_130; goto block_120; @@ -57796,8 +57796,8 @@ case 5: { lean_object* x_131; x_131 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__38; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_131; goto block_120; @@ -57806,8 +57806,8 @@ case 6: { lean_object* x_132; x_132 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__42; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_132; goto block_120; @@ -57816,8 +57816,8 @@ case 7: { lean_object* x_133; x_133 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__46; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_133; goto block_120; @@ -57826,8 +57826,8 @@ case 8: { lean_object* x_134; x_134 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__50; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_134; goto block_120; @@ -57836,8 +57836,8 @@ case 9: { lean_object* x_135; x_135 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__54; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_135; goto block_120; @@ -57846,8 +57846,8 @@ case 10: { lean_object* x_136; x_136 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__58; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_136; goto block_120; @@ -57856,8 +57856,8 @@ goto block_120; { lean_object* x_137; x_137 = l_Lean_Lsp_Ipc_readResponseAs___at___00Lean_Server_Test_Runner_request___at___00Lean_Server_Test_Runner_rpcRequest___at___00Lean_Server_Test_Runner_expandTraces_spec__2_spec__3_spec__5___closed__62; -x_94 = x_124; -x_95 = x_123; +x_94 = x_123; +x_95 = x_124; x_96 = x_125; x_97 = x_137; goto block_120; @@ -58265,7 +58265,7 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Server_Test_Runner_main(lean_object* x_1) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_31; lean_object* x_32; lean_object* x_45; uint8_t x_46; +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_31; lean_object* x_32; lean_object* x_45; uint8_t x_46; x_3 = lean_array_mk(x_1); x_4 = lean_unsigned_to_nat(0u); x_45 = lean_array_get_size(x_3); @@ -58300,7 +58300,7 @@ goto block_41; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; x_10 = l_Lean_Server_Test_Runner_main___closed__0; x_11 = lean_string_append(x_10, x_9); -x_12 = lean_box(x_6); +x_12 = lean_box(x_8); x_13 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_13, 0, x_12); x_14 = lean_box(0); @@ -58341,7 +58341,7 @@ x_26 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_23); lean_ctor_set(x_26, 2, x_25); -x_27 = lean_box(x_6); +x_27 = lean_box(x_8); x_28 = lean_alloc_closure((void*)(l_Lean_Server_Test_Runner_main___lam__1___boxed), 9, 7); lean_closure_set(x_28, 0, x_26); lean_closure_set(x_28, 1, x_22); @@ -58350,7 +58350,7 @@ lean_closure_set(x_28, 3, x_4); lean_closure_set(x_28, 4, x_11); lean_closure_set(x_28, 5, x_27); lean_closure_set(x_28, 6, x_7); -x_29 = l_Lean_Lsp_Ipc_runWith___redArg(x_5, x_8, x_28); +x_29 = l_Lean_Lsp_Ipc_runWith___redArg(x_6, x_5, x_28); return x_29; } block_41: @@ -58366,10 +58366,10 @@ lean_object* x_37; lean_object* x_38; x_37 = l_Lean_Server_Test_Runner_word___closed__0; x_38 = lean_array_get(x_37, x_3, x_34); lean_dec_ref(x_3); -x_5 = x_31; -x_6 = x_36; +x_5 = x_32; +x_6 = x_31; x_7 = x_34; -x_8 = x_32; +x_8 = x_36; x_9 = x_38; goto block_30; } @@ -58379,10 +58379,10 @@ lean_object* x_39; lean_object* x_40; x_39 = l_Lean_Server_Test_Runner_word___closed__0; x_40 = lean_array_get(x_39, x_3, x_4); lean_dec_ref(x_3); -x_5 = x_31; -x_6 = x_36; +x_5 = x_32; +x_6 = x_31; x_7 = x_34; -x_8 = x_32; +x_8 = x_36; x_9 = x_40; goto block_30; } diff --git a/stage0/stdlib/Lean/Server/Watchdog.c b/stage0/stdlib/Lean/Server/Watchdog.c index 1c617dc67b6e..63e9b61d74dc 100644 --- a/stage0/stdlib/Lean/Server/Watchdog.c +++ b/stage0/stdlib/Lean/Server/Watchdog.c @@ -49859,9 +49859,9 @@ if (x_67 == 0) uint8_t x_68; lean_object* x_69; x_68 = 11; x_69 = l_Lean_Server_Watchdog_mainLoop___closed__5; -x_23 = lean_box(0); -x_24 = x_57; -x_25 = x_58; +x_23 = x_57; +x_24 = x_58; +x_25 = lean_box(0); x_26 = x_64; x_27 = x_68; x_28 = x_69; @@ -49872,9 +49872,9 @@ else uint8_t x_70; lean_object* x_71; x_70 = 10; x_71 = l_Lean_Server_Watchdog_mainLoop___closed__6; -x_23 = lean_box(0); -x_24 = x_57; -x_25 = x_58; +x_23 = x_57; +x_24 = x_58; +x_25 = lean_box(0); x_26 = x_64; x_27 = x_70; x_28 = x_71; @@ -50246,7 +50246,7 @@ return x_6; { lean_object* x_12; lean_object* x_13; x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_9); +lean_ctor_set(x_12, 0, x_10); lean_ctor_set(x_12, 1, x_11); lean_inc_ref(x_2); x_13 = l_Lean_Server_Watchdog_writeMessage(x_12, x_2); @@ -50256,7 +50256,7 @@ uint8_t x_14; lean_object* x_15; lean_dec_ref(x_13); x_14 = 0; lean_inc_ref(x_2); -x_15 = l_Lean_Server_Watchdog_setWorkerState(x_8, x_14, x_2); +x_15 = l_Lean_Server_Watchdog_setWorkerState(x_9, x_14, x_2); if (lean_obj_tag(x_15) == 0) { lean_dec_ref(x_15); @@ -50271,7 +50271,7 @@ return x_15; } else { -lean_dec_ref(x_8); +lean_dec_ref(x_9); lean_dec_ref(x_2); lean_dec_ref(x_1); return x_13; @@ -50295,7 +50295,7 @@ if (lean_obj_tag(x_36) == 0) uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_dec_ref(x_36); x_37 = 1; -x_38 = l_Lean_Server_mkFileProgressAtPosNotification(x_25, x_22, x_37); +x_38 = l_Lean_Server_mkFileProgressAtPosNotification(x_24, x_22, x_37); x_39 = lean_ctor_get(x_38, 0); lean_inc_ref(x_39); x_40 = lean_ctor_get(x_38, 1); @@ -50307,9 +50307,9 @@ if (lean_obj_tag(x_41) == 0) lean_object* x_42; lean_dec_ref(x_41); x_42 = lean_box(0); -x_8 = x_24; -x_9 = x_39; -x_10 = lean_box(0); +x_8 = lean_box(0); +x_9 = x_23; +x_10 = x_39; x_11 = x_42; goto block_17; } @@ -50319,9 +50319,9 @@ uint8_t x_43; x_43 = !lean_is_exclusive(x_41); if (x_43 == 0) { -x_8 = x_24; -x_9 = x_39; -x_10 = lean_box(0); +x_8 = lean_box(0); +x_9 = x_23; +x_10 = x_39; x_11 = x_41; goto block_17; } @@ -50333,9 +50333,9 @@ lean_inc(x_44); lean_dec(x_41); x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_44); -x_8 = x_24; -x_9 = x_39; -x_10 = lean_box(0); +x_8 = lean_box(0); +x_9 = x_23; +x_10 = x_39; x_11 = x_45; goto block_17; } @@ -50343,8 +50343,8 @@ goto block_17; } else { -lean_dec_ref(x_25); lean_dec_ref(x_24); +lean_dec_ref(x_23); lean_dec_ref(x_2); lean_dec_ref(x_1); return x_36; @@ -51661,7 +51661,7 @@ goto block_138; { 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; x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_102); +lean_ctor_set(x_106, 0, x_103); lean_ctor_set(x_106, 1, x_105); x_107 = l_Lean_Server_Watchdog_parseRequestParams_x3f___redArg___closed__12; x_108 = lean_alloc_ctor(3, 1, 0); @@ -51682,13 +51682,13 @@ lean_dec(x_101); x_115 = l_List_appendTR___redArg(x_112, x_114); x_116 = l_Lean_Json_mkObj(x_115); x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_103); +lean_ctor_set(x_117, 0, x_104); lean_ctor_set(x_117, 1, x_116); x_118 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_118, 0, x_117); lean_ctor_set(x_118, 1, x_110); x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_104); +lean_ctor_set(x_119, 0, x_102); lean_ctor_set(x_119, 1, x_118); x_39 = x_119; goto block_48; @@ -51706,9 +51706,9 @@ case 0: { lean_object* x_126; x_126 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__5; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_126; goto block_120; } @@ -51716,9 +51716,9 @@ case 1: { lean_object* x_127; x_127 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__7; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_127; goto block_120; } @@ -51726,9 +51726,9 @@ case 2: { lean_object* x_128; x_128 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__9; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_128; goto block_120; } @@ -51736,9 +51736,9 @@ case 3: { lean_object* x_129; x_129 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__11; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_129; goto block_120; } @@ -51746,9 +51746,9 @@ case 4: { lean_object* x_130; x_130 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__13; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_130; goto block_120; } @@ -51756,9 +51756,9 @@ case 5: { lean_object* x_131; x_131 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__15; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_131; goto block_120; } @@ -51766,9 +51766,9 @@ case 6: { lean_object* x_132; x_132 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__17; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_132; goto block_120; } @@ -51776,9 +51776,9 @@ case 7: { lean_object* x_133; x_133 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__19; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_133; goto block_120; } @@ -51786,9 +51786,9 @@ case 8: { lean_object* x_134; x_134 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__21; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_134; goto block_120; } @@ -51796,9 +51796,9 @@ case 9: { lean_object* x_135; x_135 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__23; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_135; goto block_120; } @@ -51806,9 +51806,9 @@ case 10: { lean_object* x_136; x_136 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__25; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_136; goto block_120; } @@ -51816,9 +51816,9 @@ goto block_120; { lean_object* x_137; x_137 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__27; -x_102 = x_125; -x_103 = x_124; -x_104 = x_123; +x_102 = x_123; +x_103 = x_125; +x_104 = x_124; x_105 = x_137; goto block_120; } @@ -53492,7 +53492,7 @@ goto block_32; } else { -uint8_t x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_44; lean_object* x_45; lean_object* x_51; +uint8_t x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_44; lean_object* x_45; lean_object* x_51; x_36 = lean_ctor_get_uint8(x_33, sizeof(void*)*1); x_37 = lean_ctor_get(x_33, 0); lean_inc_ref(x_37); @@ -53683,8 +53683,8 @@ lean_dec_ref(x_72); x_73 = lean_box(0); x_74 = lean_unbox(x_67); lean_dec(x_67); -x_38 = x_70; -x_39 = x_74; +x_38 = x_74; +x_39 = x_70; x_40 = x_61; x_41 = x_73; goto block_43; @@ -53698,8 +53698,8 @@ if (x_75 == 0) uint8_t x_76; x_76 = lean_unbox(x_67); lean_dec(x_67); -x_38 = x_70; -x_39 = x_76; +x_38 = x_76; +x_39 = x_70; x_40 = x_61; x_41 = x_72; goto block_43; @@ -53714,8 +53714,8 @@ x_78 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_78, 0, x_77); x_79 = lean_unbox(x_67); lean_dec(x_67); -x_38 = x_70; -x_39 = x_79; +x_38 = x_79; +x_39 = x_70; x_40 = x_61; x_41 = x_78; goto block_43; @@ -53828,9 +53828,9 @@ goto block_50; lean_object* x_42; x_42 = lean_alloc_ctor(3, 3, 1); lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_38); +lean_ctor_set(x_42, 1, x_39); lean_ctor_set(x_42, 2, x_41); -lean_ctor_set_uint8(x_42, sizeof(void*)*3, x_39); +lean_ctor_set_uint8(x_42, sizeof(void*)*3, x_38); x_14 = x_36; x_15 = x_42; goto block_32; @@ -53858,7 +53858,7 @@ goto block_32; block_12: { lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00Lean_Server_Watchdog_runMessageLoggingTask_spec__0___redArg(x_5, x_7, x_9); +x_10 = l_Std_DHashMap_Internal_Raw_u2080_insert___at___00Lean_Server_Watchdog_runMessageLoggingTask_spec__0___redArg(x_5, x_8, x_9); x_5 = x_10; goto _start; } @@ -53882,8 +53882,8 @@ if (lean_obj_tag(x_18) == 0) lean_object* x_19; lean_object* x_20; x_19 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00Lean_Server_Watchdog_handleModuleHierarchyImports_spec__2___closed__3; x_20 = l_panic___at___00Lean_Server_Watchdog_runMessageLoggingTask_spec__1(x_19); -x_7 = x_17; -x_8 = lean_box(0); +x_7 = lean_box(0); +x_8 = x_17; x_9 = x_20; goto block_12; } @@ -53893,8 +53893,8 @@ lean_object* x_21; x_21 = lean_ctor_get(x_18, 0); lean_inc(x_21); lean_dec_ref(x_18); -x_7 = x_17; -x_8 = lean_box(0); +x_7 = lean_box(0); +x_8 = x_17; x_9 = x_21; goto block_12; } @@ -54742,7 +54742,7 @@ return x_36; } else { -lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_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; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_86; lean_object* x_87; lean_object* x_88; uint8_t x_94; lean_object* x_102; lean_object* x_103; +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; 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; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_86; lean_object* x_87; lean_object* x_88; uint8_t x_94; lean_object* x_102; lean_object* x_103; x_37 = lean_ctor_get(x_24, 0); lean_inc(x_37); lean_dec_ref(x_24); @@ -54784,13 +54784,13 @@ goto block_101; { lean_object* x_44; lean_object* x_45; lean_object* x_46; x_44 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_44, 0, x_40); +lean_ctor_set(x_44, 0, x_41); lean_ctor_set(x_44, 1, x_39); -lean_ctor_set(x_44, 2, x_42); -lean_ctor_set(x_44, 3, x_41); +lean_ctor_set(x_44, 2, x_38); +lean_ctor_set(x_44, 3, x_42); lean_ctor_set(x_44, 4, x_37); lean_ctor_set(x_44, 5, x_43); -lean_ctor_set_uint8(x_44, sizeof(void*)*6, x_38); +lean_ctor_set_uint8(x_44, sizeof(void*)*6, x_40); if (lean_is_scalar(x_11)) { x_45 = lean_alloc_ctor(0, 3, 0); } else { @@ -54809,46 +54809,46 @@ return x_46; } block_58: { -if (lean_obj_tag(x_51) == 0) +if (lean_obj_tag(x_52) == 0) { lean_object* x_54; -lean_dec_ref(x_51); +lean_dec_ref(x_52); x_54 = lean_box(0); -x_38 = x_48; -x_39 = x_50; -x_40 = x_49; -x_41 = x_53; -x_42 = x_52; +x_38 = x_49; +x_39 = x_48; +x_40 = x_50; +x_41 = x_51; +x_42 = x_53; x_43 = x_54; goto block_47; } else { uint8_t x_55; -x_55 = !lean_is_exclusive(x_51); +x_55 = !lean_is_exclusive(x_52); if (x_55 == 0) { -x_38 = x_48; -x_39 = x_50; -x_40 = x_49; -x_41 = x_53; -x_42 = x_52; -x_43 = x_51; +x_38 = x_49; +x_39 = x_48; +x_40 = x_50; +x_41 = x_51; +x_42 = x_53; +x_43 = x_52; goto block_47; } else { lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_51, 0); +x_56 = lean_ctor_get(x_52, 0); lean_inc(x_56); -lean_dec(x_51); +lean_dec(x_52); x_57 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_57, 0, x_56); -x_38 = x_48; -x_39 = x_50; -x_40 = x_49; -x_41 = x_53; -x_42 = x_52; +x_38 = x_49; +x_39 = x_48; +x_40 = x_50; +x_41 = x_51; +x_42 = x_53; x_43 = x_57; goto block_47; } @@ -54862,10 +54862,10 @@ lean_object* x_72; lean_dec_ref(x_66); x_72 = lean_box(0); x_48 = x_67; -x_49 = x_69; +x_49 = x_71; x_50 = x_68; -x_51 = x_70; -x_52 = x_71; +x_51 = x_69; +x_52 = x_70; x_53 = x_72; goto block_58; } @@ -54876,10 +54876,10 @@ x_73 = !lean_is_exclusive(x_66); if (x_73 == 0) { x_48 = x_67; -x_49 = x_69; +x_49 = x_71; x_50 = x_68; -x_51 = x_70; -x_52 = x_71; +x_51 = x_69; +x_52 = x_70; x_53 = x_66; goto block_58; } @@ -54892,10 +54892,10 @@ lean_dec(x_66); x_75 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_75, 0, x_74); x_48 = x_67; -x_49 = x_69; +x_49 = x_71; x_50 = x_68; -x_51 = x_70; -x_52 = x_71; +x_51 = x_69; +x_52 = x_70; x_53 = x_75; goto block_58; } @@ -54908,8 +54908,8 @@ if (lean_obj_tag(x_64) == 0) lean_object* x_81; lean_dec_ref(x_64); x_81 = lean_box(0); -x_67 = x_77; -x_68 = x_80; +x_67 = x_80; +x_68 = x_77; x_69 = x_78; x_70 = x_79; x_71 = x_81; @@ -54921,8 +54921,8 @@ uint8_t x_82; x_82 = !lean_is_exclusive(x_64); if (x_82 == 0) { -x_67 = x_77; -x_68 = x_80; +x_67 = x_80; +x_68 = x_77; x_69 = x_78; x_70 = x_79; x_71 = x_64; @@ -54936,8 +54936,8 @@ lean_inc(x_83); lean_dec(x_64); x_84 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_84, 0, x_83); -x_67 = x_77; -x_68 = x_80; +x_67 = x_80; +x_68 = x_77; x_69 = x_78; x_70 = x_79; x_71 = x_84; @@ -55301,7 +55301,7 @@ goto block_208; { 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; x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_172); +lean_ctor_set(x_176, 0, x_173); lean_ctor_set(x_176, 1, x_175); x_177 = l_Lean_Server_Watchdog_parseRequestParams_x3f___redArg___closed__12; x_178 = lean_alloc_ctor(3, 1, 0); @@ -55322,13 +55322,13 @@ lean_dec(x_171); x_185 = l_List_appendTR___redArg(x_182, x_184); x_186 = l_Lean_Json_mkObj(x_185); x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_173); +lean_ctor_set(x_187, 0, x_174); lean_ctor_set(x_187, 1, x_186); x_188 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_188, 0, x_187); lean_ctor_set(x_188, 1, x_180); x_189 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_189, 0, x_174); +lean_ctor_set(x_189, 0, x_172); lean_ctor_set(x_189, 1, x_188); x_109 = x_189; goto block_118; @@ -55346,9 +55346,9 @@ case 0: { lean_object* x_196; x_196 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__5; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_196; goto block_190; } @@ -55356,9 +55356,9 @@ case 1: { lean_object* x_197; x_197 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__7; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_197; goto block_190; } @@ -55366,9 +55366,9 @@ case 2: { lean_object* x_198; x_198 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__9; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_198; goto block_190; } @@ -55376,9 +55376,9 @@ case 3: { lean_object* x_199; x_199 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__11; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_199; goto block_190; } @@ -55386,9 +55386,9 @@ case 4: { lean_object* x_200; x_200 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__13; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_200; goto block_190; } @@ -55396,9 +55396,9 @@ case 5: { lean_object* x_201; x_201 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__15; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_201; goto block_190; } @@ -55406,9 +55406,9 @@ case 6: { lean_object* x_202; x_202 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__17; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_202; goto block_190; } @@ -55416,9 +55416,9 @@ case 7: { lean_object* x_203; x_203 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__19; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_203; goto block_190; } @@ -55426,9 +55426,9 @@ case 8: { lean_object* x_204; x_204 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__21; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_204; goto block_190; } @@ -55436,9 +55436,9 @@ case 9: { lean_object* x_205; x_205 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__23; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_205; goto block_190; } @@ -55446,9 +55446,9 @@ case 10: { lean_object* x_206; x_206 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__25; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_206; goto block_190; } @@ -55456,9 +55456,9 @@ goto block_190; { lean_object* x_207; x_207 = l_IO_FS_Stream_readNotificationAs___at___00IO_FS_Stream_readLspNotificationAs___at___00Lean_Server_Watchdog_initAndRunWatchdogAux_spec__1_spec__1___closed__27; -x_172 = x_195; -x_173 = x_194; -x_174 = x_193; +x_172 = x_193; +x_173 = x_195; +x_174 = x_194; x_175 = x_207; goto block_190; } diff --git a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c index efb7382f52b5..ad756757d7f2 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c +++ b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c @@ -6947,14 +6947,14 @@ if (lean_is_scalar(x_15)) { x_30 = x_15; } lean_ctor_set(x_30, 0, x_19); -lean_ctor_set(x_30, 1, x_25); -lean_ctor_set(x_30, 2, x_24); -lean_ctor_set(x_30, 3, x_22); -lean_ctor_set(x_30, 4, x_23); -lean_ctor_set(x_30, 5, x_26); -lean_ctor_set(x_30, 6, x_20); -lean_ctor_set(x_30, 7, x_21); -lean_ctor_set(x_30, 8, x_27); +lean_ctor_set(x_30, 1, x_24); +lean_ctor_set(x_30, 2, x_22); +lean_ctor_set(x_30, 3, x_25); +lean_ctor_set(x_30, 4, x_21); +lean_ctor_set(x_30, 5, x_27); +lean_ctor_set(x_30, 6, x_26); +lean_ctor_set(x_30, 7, x_20); +lean_ctor_set(x_30, 8, x_23); lean_ctor_set(x_30, 9, x_28); lean_ctor_set(x_30, 10, x_14); x_31 = l_Lean_Widget_instToJsonRpcEncodablePacket_toJson_00___x40_Lean_Widget_InteractiveDiagnostic_3833933514____hygCtx___hyg_123_(x_30); @@ -6976,11 +6976,11 @@ x_44 = lean_box(0); x_20 = x_34; x_21 = x_35; x_22 = x_36; -x_23 = x_37; -x_24 = x_39; +x_23 = x_41; +x_24 = x_37; x_25 = x_38; -x_26 = x_40; -x_27 = x_41; +x_26 = x_39; +x_27 = x_40; x_28 = x_44; x_29 = x_42; goto block_33; @@ -7008,11 +7008,11 @@ lean_ctor_set(x_13, 0, x_54); x_20 = x_34; x_21 = x_35; x_22 = x_36; -x_23 = x_37; -x_24 = x_39; +x_23 = x_41; +x_24 = x_37; x_25 = x_38; -x_26 = x_40; -x_27 = x_41; +x_26 = x_39; +x_27 = x_40; x_28 = x_13; x_29 = x_52; goto block_33; @@ -7039,11 +7039,11 @@ lean_ctor_set(x_64, 0, x_63); x_20 = x_34; x_21 = x_35; x_22 = x_36; -x_23 = x_37; -x_24 = x_39; +x_23 = x_41; +x_24 = x_37; x_25 = x_38; -x_26 = x_40; -x_27 = x_41; +x_26 = x_39; +x_27 = x_40; x_28 = x_64; x_29 = x_61; goto block_33; @@ -7059,12 +7059,12 @@ if (lean_obj_tag(x_12) == 0) lean_object* x_75; lean_dec_ref(x_16); x_75 = lean_box(0); -x_34 = x_66; -x_35 = x_72; +x_34 = x_72; +x_35 = x_66; x_36 = x_67; x_37 = x_68; -x_38 = x_70; -x_39 = x_69; +x_38 = x_69; +x_39 = x_70; x_40 = x_71; x_41 = x_75; x_42 = x_73; @@ -7090,12 +7090,12 @@ lean_dec_ref(x_81); x_84 = l_Lean_Widget_instRpcEncodableDiagnosticWith_enc___redArg___closed__20_00___x40_Lean_Widget_InteractiveDiagnostic_2989700264____hygCtx___hyg_2_; x_85 = l_Array_toJson___redArg(x_84, x_82); lean_ctor_set(x_12, 0, x_85); -x_34 = x_66; -x_35 = x_72; +x_34 = x_72; +x_35 = x_66; x_36 = x_67; x_37 = x_68; -x_38 = x_70; -x_39 = x_69; +x_38 = x_69; +x_39 = x_70; x_40 = x_71; x_41 = x_12; x_42 = x_83; @@ -7120,12 +7120,12 @@ x_93 = l_Lean_Widget_instRpcEncodableDiagnosticWith_enc___redArg___closed__20_00 x_94 = l_Array_toJson___redArg(x_93, x_91); x_95 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_95, 0, x_94); -x_34 = x_66; -x_35 = x_72; +x_34 = x_72; +x_35 = x_66; x_36 = x_67; x_37 = x_68; -x_38 = x_70; -x_39 = x_69; +x_38 = x_69; +x_39 = x_70; x_40 = x_71; x_41 = x_95; x_42 = x_92; @@ -7151,11 +7151,11 @@ if (lean_obj_tag(x_11) == 0) lean_object* x_108; lean_dec_ref(x_18); x_108 = lean_box(0); -x_66 = x_105; -x_67 = x_97; -x_68 = x_98; +x_66 = x_97; +x_67 = x_98; +x_68 = x_99; x_69 = x_100; -x_70 = x_99; +x_70 = x_105; x_71 = x_101; x_72 = x_108; x_73 = x_106; @@ -7181,11 +7181,11 @@ lean_dec_ref(x_114); x_117 = l_Lean_Widget_instRpcEncodableDiagnosticWith_enc___redArg___closed__20_00___x40_Lean_Widget_InteractiveDiagnostic_2989700264____hygCtx___hyg_2_; x_118 = l_Array_toJson___redArg(x_117, x_115); lean_ctor_set(x_11, 0, x_118); -x_66 = x_105; -x_67 = x_97; -x_68 = x_98; +x_66 = x_97; +x_67 = x_98; +x_68 = x_99; x_69 = x_100; -x_70 = x_99; +x_70 = x_105; x_71 = x_101; x_72 = x_11; x_73 = x_116; @@ -7210,11 +7210,11 @@ x_126 = l_Lean_Widget_instRpcEncodableDiagnosticWith_enc___redArg___closed__20_0 x_127 = l_Array_toJson___redArg(x_126, x_124); x_128 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_128, 0, x_127); -x_66 = x_105; -x_67 = x_97; -x_68 = x_98; +x_66 = x_97; +x_67 = x_98; +x_68 = x_99; x_69 = x_100; -x_70 = x_99; +x_70 = x_105; x_71 = x_101; x_72 = x_128; x_73 = x_125; @@ -7228,10 +7228,10 @@ if (lean_obj_tag(x_9) == 0) { lean_object* x_135; x_135 = lean_box(0); -x_97 = x_130; -x_98 = x_133; -x_99 = x_132; -x_100 = x_131; +x_97 = x_133; +x_98 = x_130; +x_99 = x_131; +x_100 = x_132; x_101 = x_135; x_102 = x_134; goto block_129; @@ -7247,10 +7247,10 @@ x_137 = lean_ctor_get(x_9, 0); x_138 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_138, 0, x_137); lean_ctor_set(x_9, 0, x_138); -x_97 = x_130; -x_98 = x_133; -x_99 = x_132; -x_100 = x_131; +x_97 = x_133; +x_98 = x_130; +x_99 = x_131; +x_100 = x_132; x_101 = x_9; x_102 = x_134; goto block_129; @@ -7265,10 +7265,10 @@ x_140 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_140, 0, x_139); x_141 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_141, 0, x_140); -x_97 = x_130; -x_98 = x_133; -x_99 = x_132; -x_100 = x_131; +x_97 = x_133; +x_98 = x_130; +x_99 = x_131; +x_100 = x_132; x_101 = x_141; x_102 = x_134; goto block_129; @@ -7281,8 +7281,8 @@ lean_object* x_148; x_148 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_148, 0, x_146); x_130 = x_143; -x_131 = x_145; -x_132 = x_144; +x_131 = x_144; +x_132 = x_145; x_133 = x_148; x_134 = x_147; goto block_142; @@ -7293,9 +7293,9 @@ if (lean_obj_tag(x_8) == 0) { lean_object* x_154; x_154 = lean_box(0); -x_130 = x_152; +x_130 = x_150; x_131 = x_151; -x_132 = x_150; +x_132 = x_152; x_133 = x_154; x_134 = x_153; goto block_142; @@ -7317,9 +7317,9 @@ x_157 = lean_ctor_get(x_155, 0); x_158 = l_Lean_JsonNumber_fromInt(x_157); lean_ctor_set_tag(x_155, 2); lean_ctor_set(x_155, 0, x_158); -x_143 = x_152; -x_144 = x_150; -x_145 = x_151; +x_143 = x_150; +x_144 = x_151; +x_145 = x_152; x_146 = x_155; x_147 = x_153; goto block_149; @@ -7333,9 +7333,9 @@ lean_dec(x_155); x_160 = l_Lean_JsonNumber_fromInt(x_159); x_161 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_161, 0, x_160); -x_143 = x_152; -x_144 = x_150; -x_145 = x_151; +x_143 = x_150; +x_144 = x_151; +x_145 = x_152; x_146 = x_161; x_147 = x_153; goto block_149; @@ -7348,9 +7348,9 @@ x_162 = !lean_is_exclusive(x_155); if (x_162 == 0) { lean_ctor_set_tag(x_155, 3); -x_143 = x_152; -x_144 = x_150; -x_145 = x_151; +x_143 = x_150; +x_144 = x_151; +x_145 = x_152; x_146 = x_155; x_147 = x_153; goto block_149; @@ -7363,9 +7363,9 @@ lean_inc(x_163); lean_dec(x_155); x_164 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_164, 0, x_163); -x_143 = x_152; -x_144 = x_150; -x_145 = x_151; +x_143 = x_150; +x_144 = x_151; +x_145 = x_152; x_146 = x_164; x_147 = x_153; goto block_149; @@ -7379,8 +7379,8 @@ if (lean_obj_tag(x_7) == 0) { lean_object* x_169; x_169 = lean_box(0); -x_150 = x_166; -x_151 = x_167; +x_150 = x_167; +x_151 = x_166; x_152 = x_169; x_153 = x_168; goto block_165; @@ -7398,8 +7398,8 @@ x_173 = lean_unbox(x_171); lean_dec(x_171); lean_ctor_set_uint8(x_172, 0, x_173); lean_ctor_set(x_7, 0, x_172); -x_150 = x_166; -x_151 = x_167; +x_150 = x_167; +x_151 = x_166; x_152 = x_7; x_153 = x_168; goto block_165; @@ -7416,8 +7416,8 @@ lean_dec(x_174); lean_ctor_set_uint8(x_175, 0, x_176); x_177 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_177, 0, x_175); -x_150 = x_166; -x_151 = x_167; +x_150 = x_167; +x_151 = x_166; x_152 = x_177; x_153 = x_168; goto block_165; @@ -8217,15 +8217,15 @@ if (lean_is_scalar(x_30)) { x_49 = x_30; } lean_ctor_set(x_49, 0, x_37); -lean_ctor_set(x_49, 1, x_42); -lean_ctor_set(x_49, 2, x_40); -lean_ctor_set(x_49, 3, x_43); -lean_ctor_set(x_49, 4, x_47); -lean_ctor_set(x_49, 5, x_46); +lean_ctor_set(x_49, 1, x_45); +lean_ctor_set(x_49, 2, x_47); +lean_ctor_set(x_49, 3, x_40); +lean_ctor_set(x_49, 4, x_46); +lean_ctor_set(x_49, 5, x_44); lean_ctor_set(x_49, 6, x_41); -lean_ctor_set(x_49, 7, x_45); -lean_ctor_set(x_49, 8, x_39); -lean_ctor_set(x_49, 9, x_44); +lean_ctor_set(x_49, 7, x_42); +lean_ctor_set(x_49, 8, x_43); +lean_ctor_set(x_49, 9, x_39); lean_ctor_set(x_49, 10, x_48); if (lean_is_scalar(x_38)) { x_50 = lean_alloc_ctor(1, 1, 0); @@ -8242,15 +8242,15 @@ if (lean_obj_tag(x_29) == 0) lean_dec_ref(x_61); lean_dec_ref(x_18); lean_dec(x_9); -x_39 = x_52; -x_40 = x_53; -x_41 = x_55; +x_39 = x_60; +x_40 = x_52; +x_41 = x_53; x_42 = x_54; -x_43 = x_56; -x_44 = x_60; -x_45 = x_59; -x_46 = x_58; -x_47 = x_57; +x_43 = x_55; +x_44 = x_56; +x_45 = x_57; +x_46 = x_59; +x_47 = x_58; x_48 = x_29; goto block_51; } @@ -8309,15 +8309,15 @@ x_70 = lean_ctor_get(x_66, 0); lean_inc(x_70); lean_dec_ref(x_66); lean_ctor_set(x_29, 0, x_70); -x_39 = x_52; -x_40 = x_53; -x_41 = x_55; +x_39 = x_60; +x_40 = x_52; +x_41 = x_53; x_42 = x_54; -x_43 = x_56; -x_44 = x_60; -x_45 = x_59; -x_46 = x_58; -x_47 = x_57; +x_43 = x_55; +x_44 = x_56; +x_45 = x_57; +x_46 = x_59; +x_47 = x_58; x_48 = x_29; goto block_51; } @@ -8376,15 +8376,15 @@ lean_inc(x_78); lean_dec_ref(x_74); x_79 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_79, 0, x_78); -x_39 = x_52; -x_40 = x_53; -x_41 = x_55; +x_39 = x_60; +x_40 = x_52; +x_41 = x_53; x_42 = x_54; -x_43 = x_56; -x_44 = x_60; -x_45 = x_59; -x_46 = x_58; -x_47 = x_57; +x_43 = x_55; +x_44 = x_56; +x_45 = x_57; +x_46 = x_59; +x_47 = x_58; x_48 = x_79; goto block_51; } @@ -8398,14 +8398,14 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_91; lean_dec_ref(x_81); x_91 = lean_box(0); -x_52 = x_89; -x_53 = x_82; +x_52 = x_82; +x_53 = x_83; x_54 = x_84; -x_55 = x_83; +x_55 = x_89; x_56 = x_85; -x_57 = x_88; -x_58 = x_87; -x_59 = x_86; +x_57 = x_86; +x_58 = x_88; +x_59 = x_87; x_60 = x_91; x_61 = x_90; goto block_80; @@ -8509,14 +8509,14 @@ x_107 = lean_ctor_get(x_103, 0); lean_inc(x_107); lean_dec_ref(x_103); lean_ctor_set(x_28, 0, x_107); -x_52 = x_89; -x_53 = x_82; +x_52 = x_82; +x_53 = x_83; x_54 = x_84; -x_55 = x_83; +x_55 = x_89; x_56 = x_85; -x_57 = x_88; -x_58 = x_87; -x_59 = x_86; +x_57 = x_86; +x_58 = x_88; +x_59 = x_87; x_60 = x_28; x_61 = x_90; goto block_80; @@ -8621,14 +8621,14 @@ lean_inc(x_122); lean_dec_ref(x_118); x_123 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_123, 0, x_122); -x_52 = x_89; -x_53 = x_82; +x_52 = x_82; +x_53 = x_83; x_54 = x_84; -x_55 = x_83; +x_55 = x_89; x_56 = x_85; -x_57 = x_88; -x_58 = x_87; -x_59 = x_86; +x_57 = x_86; +x_58 = x_88; +x_59 = x_87; x_60 = x_123; x_61 = x_90; goto block_80; @@ -8645,10 +8645,10 @@ lean_object* x_134; lean_dec_ref(x_125); x_134 = lean_box(0); x_82 = x_126; -x_83 = x_128; -x_84 = x_127; -x_85 = x_129; -x_86 = x_132; +x_83 = x_127; +x_84 = x_132; +x_85 = x_128; +x_86 = x_129; x_87 = x_131; x_88 = x_130; x_89 = x_134; @@ -8757,10 +8757,10 @@ lean_inc(x_150); lean_dec_ref(x_146); lean_ctor_set(x_27, 0, x_150); x_82 = x_126; -x_83 = x_128; -x_84 = x_127; -x_85 = x_129; -x_86 = x_132; +x_83 = x_127; +x_84 = x_132; +x_85 = x_128; +x_86 = x_129; x_87 = x_131; x_88 = x_130; x_89 = x_27; @@ -8870,10 +8870,10 @@ lean_dec_ref(x_161); x_166 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_166, 0, x_165); x_82 = x_126; -x_83 = x_128; -x_84 = x_127; -x_85 = x_129; -x_86 = x_132; +x_83 = x_127; +x_84 = x_132; +x_85 = x_128; +x_86 = x_129; x_87 = x_131; x_88 = x_130; x_89 = x_166; @@ -8940,11 +8940,11 @@ lean_inc(x_180); lean_dec_ref(x_176); x_181 = lean_box(0); x_126 = x_169; -x_127 = x_170; -x_128 = x_180; -x_129 = x_171; +x_127 = x_180; +x_128 = x_173; +x_129 = x_170; x_130 = x_172; -x_131 = x_173; +x_131 = x_171; x_132 = x_181; x_133 = x_174; goto block_167; @@ -9056,11 +9056,11 @@ lean_inc(x_198); lean_dec_ref(x_194); lean_ctor_set(x_26, 0, x_198); x_126 = x_169; -x_127 = x_170; -x_128 = x_182; -x_129 = x_171; +x_127 = x_182; +x_128 = x_173; +x_129 = x_170; x_130 = x_172; -x_131 = x_173; +x_131 = x_171; x_132 = x_26; x_133 = x_174; goto block_167; @@ -9170,11 +9170,11 @@ lean_dec_ref(x_209); x_214 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_214, 0, x_213); x_126 = x_169; -x_127 = x_170; -x_128 = x_182; -x_129 = x_171; +x_127 = x_182; +x_128 = x_173; +x_129 = x_170; x_130 = x_172; -x_131 = x_173; +x_131 = x_171; x_132 = x_214; x_133 = x_174; goto block_167; @@ -9192,8 +9192,8 @@ lean_object* x_221; x_221 = lean_box(0); x_169 = x_216; x_170 = x_217; -x_171 = x_218; -x_172 = x_219; +x_171 = x_219; +x_172 = x_218; x_173 = x_221; x_174 = x_220; goto block_215; @@ -9259,8 +9259,8 @@ lean_dec_ref(x_226); lean_ctor_set(x_24, 0, x_230); x_169 = x_216; x_170 = x_217; -x_171 = x_218; -x_172 = x_219; +x_171 = x_219; +x_172 = x_218; x_173 = x_24; x_174 = x_220; goto block_215; @@ -9326,8 +9326,8 @@ x_239 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_239, 0, x_238); x_169 = x_216; x_170 = x_217; -x_171 = x_218; -x_172 = x_219; +x_171 = x_219; +x_172 = x_218; x_173 = x_239; x_174 = x_220; goto block_215; @@ -9340,10 +9340,10 @@ goto block_215; if (lean_obj_tag(x_245) == 0) { uint8_t x_246; -lean_dec_ref(x_244); +lean_dec(x_244); lean_dec(x_243); lean_dec(x_242); -lean_dec(x_241); +lean_dec_ref(x_241); lean_dec_ref(x_168); lean_dec_ref(x_125); lean_dec_ref(x_81); @@ -9383,11 +9383,11 @@ lean_inc(x_249); lean_dec_ref(x_245); x_250 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_250, 0, x_249); -x_216 = x_241; -x_217 = x_242; -x_218 = x_243; +x_216 = x_242; +x_217 = x_243; +x_218 = x_244; x_219 = x_250; -x_220 = x_244; +x_220 = x_241; goto block_240; } } @@ -9405,8 +9405,8 @@ x_263 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_263, 0, x_262); lean_inc_ref(x_18); x_264 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_263); -lean_inc_ref(x_255); -x_265 = lean_apply_1(x_264, x_255); +lean_inc_ref(x_252); +x_265 = lean_apply_1(x_264, x_252); x_241 = x_252; x_242 = x_253; x_243 = x_254; @@ -9420,9 +9420,9 @@ if (lean_obj_tag(x_23) == 0) { lean_object* x_271; x_271 = lean_box(0); -x_216 = x_267; -x_217 = x_268; -x_218 = x_269; +x_216 = x_269; +x_217 = x_267; +x_218 = x_268; x_219 = x_271; x_220 = x_270; goto block_240; @@ -9447,10 +9447,10 @@ x_278 = lean_nat_dec_eq(x_276, x_277); if (x_278 == 0) { lean_free_object(x_23); -x_252 = x_267; -x_253 = x_268; -x_254 = x_269; -x_255 = x_270; +x_252 = x_270; +x_253 = x_269; +x_254 = x_267; +x_255 = x_268; x_256 = x_273; goto block_266; } @@ -9470,10 +9470,10 @@ lean_inc_ref(x_18); x_281 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_23); lean_inc_ref(x_270); x_282 = lean_apply_1(x_281, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_282; goto block_251; } @@ -9488,10 +9488,10 @@ lean_inc_ref(x_18); x_284 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_23); lean_inc_ref(x_270); x_285 = lean_apply_1(x_284, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_285; goto block_251; } @@ -9509,10 +9509,10 @@ lean_inc_ref(x_18); x_287 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_23); lean_inc_ref(x_270); x_288 = lean_apply_1(x_287, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_288; goto block_251; } @@ -9529,10 +9529,10 @@ lean_inc_ref(x_18); x_291 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_23); lean_inc_ref(x_270); x_292 = lean_apply_1(x_291, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_292; goto block_251; } @@ -9540,10 +9540,10 @@ goto block_251; default: { lean_free_object(x_23); -x_252 = x_267; -x_253 = x_268; -x_254 = x_269; -x_255 = x_270; +x_252 = x_270; +x_253 = x_269; +x_254 = x_267; +x_255 = x_268; x_256 = x_273; goto block_266; } @@ -9566,10 +9566,10 @@ x_297 = lean_unsigned_to_nat(0u); x_298 = lean_nat_dec_eq(x_296, x_297); if (x_298 == 0) { -x_252 = x_267; -x_253 = x_268; -x_254 = x_269; -x_255 = x_270; +x_252 = x_270; +x_253 = x_269; +x_254 = x_267; +x_255 = x_268; x_256 = x_293; goto block_266; } @@ -9597,10 +9597,10 @@ lean_inc_ref(x_18); x_302 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_301); lean_inc_ref(x_270); x_303 = lean_apply_1(x_302, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_303; goto block_251; } @@ -9630,19 +9630,19 @@ lean_inc_ref(x_18); x_308 = l_MonadExcept_ofExcept___redArg(x_11, x_18, x_307); lean_inc_ref(x_270); x_309 = lean_apply_1(x_308, x_270); -x_241 = x_267; -x_242 = x_268; -x_243 = x_269; -x_244 = x_270; +x_241 = x_270; +x_242 = x_269; +x_243 = x_267; +x_244 = x_268; x_245 = x_309; goto block_251; } default: { -x_252 = x_267; -x_253 = x_268; -x_254 = x_269; -x_255 = x_270; +x_252 = x_270; +x_253 = x_269; +x_254 = x_267; +x_255 = x_268; x_256 = x_293; goto block_266; } @@ -9656,8 +9656,8 @@ if (lean_obj_tag(x_22) == 0) { lean_object* x_314; x_314 = lean_box(0); -x_267 = x_312; -x_268 = x_311; +x_267 = x_311; +x_268 = x_312; x_269 = x_314; x_270 = x_313; goto block_310; @@ -9722,8 +9722,8 @@ x_323 = lean_ctor_get(x_319, 0); lean_inc(x_323); lean_dec_ref(x_319); lean_ctor_set(x_22, 0, x_323); -x_267 = x_312; -x_268 = x_311; +x_267 = x_311; +x_268 = x_312; x_269 = x_22; x_270 = x_313; goto block_310; @@ -9788,8 +9788,8 @@ lean_inc(x_331); lean_dec_ref(x_327); x_332 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_332, 0, x_331); -x_267 = x_312; -x_268 = x_311; +x_267 = x_311; +x_268 = x_312; x_269 = x_332; x_270 = x_313; goto block_310; @@ -10207,15 +10207,15 @@ if (lean_is_scalar(x_419)) { x_438 = x_419; } lean_ctor_set(x_438, 0, x_426); -lean_ctor_set(x_438, 1, x_431); -lean_ctor_set(x_438, 2, x_429); -lean_ctor_set(x_438, 3, x_432); -lean_ctor_set(x_438, 4, x_436); -lean_ctor_set(x_438, 5, x_435); +lean_ctor_set(x_438, 1, x_434); +lean_ctor_set(x_438, 2, x_436); +lean_ctor_set(x_438, 3, x_429); +lean_ctor_set(x_438, 4, x_435); +lean_ctor_set(x_438, 5, x_433); lean_ctor_set(x_438, 6, x_430); -lean_ctor_set(x_438, 7, x_434); -lean_ctor_set(x_438, 8, x_428); -lean_ctor_set(x_438, 9, x_433); +lean_ctor_set(x_438, 7, x_431); +lean_ctor_set(x_438, 8, x_432); +lean_ctor_set(x_438, 9, x_428); lean_ctor_set(x_438, 10, x_437); if (lean_is_scalar(x_427)) { x_439 = lean_alloc_ctor(1, 1, 0); @@ -10232,15 +10232,15 @@ if (lean_obj_tag(x_418) == 0) lean_dec_ref(x_450); lean_dec_ref(x_407); lean_dec(x_9); -x_428 = x_441; -x_429 = x_442; -x_430 = x_444; +x_428 = x_449; +x_429 = x_441; +x_430 = x_442; x_431 = x_443; -x_432 = x_445; -x_433 = x_449; -x_434 = x_448; -x_435 = x_447; -x_436 = x_446; +x_432 = x_444; +x_433 = x_445; +x_434 = x_446; +x_435 = x_448; +x_436 = x_447; x_437 = x_418; goto block_440; } @@ -10309,15 +10309,15 @@ if (lean_is_scalar(x_452)) { x_460 = x_452; } lean_ctor_set(x_460, 0, x_459); -x_428 = x_441; -x_429 = x_442; -x_430 = x_444; +x_428 = x_449; +x_429 = x_441; +x_430 = x_442; x_431 = x_443; -x_432 = x_445; -x_433 = x_449; -x_434 = x_448; -x_435 = x_447; -x_436 = x_446; +x_432 = x_444; +x_433 = x_445; +x_434 = x_446; +x_435 = x_448; +x_436 = x_447; x_437 = x_460; goto block_440; } @@ -10330,14 +10330,14 @@ if (lean_obj_tag(x_417) == 0) lean_object* x_472; lean_dec_ref(x_462); x_472 = lean_box(0); -x_441 = x_470; -x_442 = x_463; +x_441 = x_463; +x_442 = x_464; x_443 = x_465; -x_444 = x_464; +x_444 = x_470; x_445 = x_466; -x_446 = x_469; -x_447 = x_468; -x_448 = x_467; +x_446 = x_467; +x_447 = x_469; +x_448 = x_468; x_449 = x_472; x_450 = x_471; goto block_461; @@ -10452,14 +10452,14 @@ if (lean_is_scalar(x_474)) { x_489 = x_474; } lean_ctor_set(x_489, 0, x_488); -x_441 = x_470; -x_442 = x_463; +x_441 = x_463; +x_442 = x_464; x_443 = x_465; -x_444 = x_464; +x_444 = x_470; x_445 = x_466; -x_446 = x_469; -x_447 = x_468; -x_448 = x_467; +x_446 = x_467; +x_447 = x_469; +x_448 = x_468; x_449 = x_489; x_450 = x_471; goto block_461; @@ -10475,10 +10475,10 @@ lean_object* x_500; lean_dec_ref(x_491); x_500 = lean_box(0); x_463 = x_492; -x_464 = x_494; -x_465 = x_493; -x_466 = x_495; -x_467 = x_498; +x_464 = x_493; +x_465 = x_498; +x_466 = x_494; +x_467 = x_495; x_468 = x_497; x_469 = x_496; x_470 = x_500; @@ -10598,10 +10598,10 @@ if (lean_is_scalar(x_502)) { } lean_ctor_set(x_517, 0, x_516); x_463 = x_492; -x_464 = x_494; -x_465 = x_493; -x_466 = x_495; -x_467 = x_498; +x_464 = x_493; +x_465 = x_498; +x_466 = x_494; +x_467 = x_495; x_468 = x_497; x_469 = x_496; x_470 = x_517; @@ -10668,11 +10668,11 @@ lean_inc(x_531); lean_dec_ref(x_527); x_532 = lean_box(0); x_492 = x_520; -x_493 = x_521; -x_494 = x_531; -x_495 = x_522; +x_493 = x_531; +x_494 = x_524; +x_495 = x_521; x_496 = x_523; -x_497 = x_524; +x_497 = x_522; x_498 = x_532; x_499 = x_525; goto block_518; @@ -10795,11 +10795,11 @@ if (lean_is_scalar(x_535)) { } lean_ctor_set(x_550, 0, x_549); x_492 = x_520; -x_493 = x_521; -x_494 = x_533; -x_495 = x_522; +x_493 = x_533; +x_494 = x_524; +x_495 = x_521; x_496 = x_523; -x_497 = x_524; +x_497 = x_522; x_498 = x_550; x_499 = x_525; goto block_518; @@ -10816,8 +10816,8 @@ lean_object* x_557; x_557 = lean_box(0); x_520 = x_552; x_521 = x_553; -x_522 = x_554; -x_523 = x_555; +x_522 = x_555; +x_523 = x_554; x_524 = x_557; x_525 = x_556; goto block_551; @@ -10893,8 +10893,8 @@ if (lean_is_scalar(x_559)) { lean_ctor_set(x_567, 0, x_566); x_520 = x_552; x_521 = x_553; -x_522 = x_554; -x_523 = x_555; +x_522 = x_555; +x_523 = x_554; x_524 = x_567; x_525 = x_556; goto block_551; @@ -10906,10 +10906,10 @@ goto block_551; if (lean_obj_tag(x_573) == 0) { lean_object* x_574; lean_object* x_575; lean_object* x_576; -lean_dec_ref(x_572); +lean_dec(x_572); lean_dec(x_571); lean_dec(x_570); -lean_dec(x_569); +lean_dec_ref(x_569); lean_dec_ref(x_519); lean_dec_ref(x_491); lean_dec_ref(x_462); @@ -10950,11 +10950,11 @@ lean_inc(x_577); lean_dec_ref(x_573); x_578 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_578, 0, x_577); -x_552 = x_569; -x_553 = x_570; -x_554 = x_571; +x_552 = x_570; +x_553 = x_571; +x_554 = x_572; x_555 = x_578; -x_556 = x_572; +x_556 = x_569; goto block_568; } } @@ -10972,8 +10972,8 @@ x_591 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_591, 0, x_590); lean_inc_ref(x_407); x_592 = l_MonadExcept_ofExcept___redArg(x_11, x_407, x_591); -lean_inc_ref(x_583); -x_593 = lean_apply_1(x_592, x_583); +lean_inc_ref(x_580); +x_593 = lean_apply_1(x_592, x_580); x_569 = x_580; x_570 = x_581; x_571 = x_582; @@ -10987,9 +10987,9 @@ if (lean_obj_tag(x_412) == 0) { lean_object* x_599; x_599 = lean_box(0); -x_552 = x_595; -x_553 = x_596; -x_554 = x_597; +x_552 = x_597; +x_553 = x_595; +x_554 = x_596; x_555 = x_599; x_556 = x_598; goto block_568; @@ -11018,10 +11018,10 @@ x_606 = lean_nat_dec_eq(x_604, x_605); if (x_606 == 0) { lean_dec(x_601); -x_580 = x_595; -x_581 = x_596; -x_582 = x_597; -x_583 = x_598; +x_580 = x_598; +x_581 = x_597; +x_582 = x_595; +x_583 = x_596; x_584 = x_600; goto block_594; } @@ -11053,10 +11053,10 @@ lean_inc_ref(x_407); x_610 = l_MonadExcept_ofExcept___redArg(x_11, x_407, x_609); lean_inc_ref(x_598); x_611 = lean_apply_1(x_610, x_598); -x_569 = x_595; -x_570 = x_596; -x_571 = x_597; -x_572 = x_598; +x_569 = x_598; +x_570 = x_597; +x_571 = x_595; +x_572 = x_596; x_573 = x_611; goto block_579; } @@ -11090,20 +11090,20 @@ lean_inc_ref(x_407); x_616 = l_MonadExcept_ofExcept___redArg(x_11, x_407, x_615); lean_inc_ref(x_598); x_617 = lean_apply_1(x_616, x_598); -x_569 = x_595; -x_570 = x_596; -x_571 = x_597; -x_572 = x_598; +x_569 = x_598; +x_570 = x_597; +x_571 = x_595; +x_572 = x_596; x_573 = x_617; goto block_579; } default: { lean_dec(x_601); -x_580 = x_595; -x_581 = x_596; -x_582 = x_597; -x_583 = x_598; +x_580 = x_598; +x_581 = x_597; +x_582 = x_595; +x_583 = x_596; x_584 = x_600; goto block_594; } @@ -11116,8 +11116,8 @@ if (lean_obj_tag(x_411) == 0) { lean_object* x_622; x_622 = lean_box(0); -x_595 = x_620; -x_596 = x_619; +x_595 = x_619; +x_596 = x_620; x_597 = x_622; x_598 = x_621; goto block_618; @@ -11192,8 +11192,8 @@ if (lean_is_scalar(x_624)) { x_632 = x_624; } lean_ctor_set(x_632, 0, x_631); -x_595 = x_620; -x_596 = x_619; +x_595 = x_619; +x_596 = x_620; x_597 = x_632; x_598 = x_621; goto block_618; @@ -12433,7 +12433,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_119; uint8_t x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_129; lean_object* x_130; lean_object* x_131; double x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; double x_137; lean_object* x_138; 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_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; 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_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_76; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_129; uint8_t x_130; double x_131; lean_object* x_132; lean_object* x_133; double x_134; uint8_t x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; 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_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; x_317 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__6; if (lean_obj_tag(x_2) == 0) { @@ -12618,9 +12618,9 @@ lean_inc_ref(x_366); lean_dec_ref(x_3); x_367 = lean_box(0); x_318 = x_4; -x_319 = x_366; +x_319 = x_2; x_320 = lean_box(0); -x_321 = x_2; +x_321 = x_366; x_322 = x_367; goto block_329; } @@ -13054,9 +13054,9 @@ x_456 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_mkPPContext x_457 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_457, 0, x_456); x_318 = x_4; -x_319 = x_455; +x_319 = x_2; x_320 = lean_box(0); -x_321 = x_2; +x_321 = x_455; x_322 = x_457; goto block_329; } @@ -13149,10 +13149,10 @@ return x_11; { lean_object* x_38; lean_object* x_39; x_38 = lean_alloc_ctor(3, 3, 1); -lean_ctor_set(x_38, 0, x_34); -lean_ctor_set(x_38, 1, x_33); +lean_ctor_set(x_38, 0, x_32); +lean_ctor_set(x_38, 1, x_34); lean_ctor_set(x_38, 2, x_35); -lean_ctor_set_uint8(x_38, sizeof(void*)*3, x_32); +lean_ctor_set_uint8(x_38, sizeof(void*)*3, x_33); x_39 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_pushEmbed(x_38, x_36); if (lean_obj_tag(x_39) == 0) { @@ -13251,18 +13251,18 @@ return x_61; { lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; x_70 = lean_unsigned_to_nat(0u); -x_71 = lean_array_get_size(x_66); -x_72 = l_Array_toSubarray___redArg(x_66, x_70, x_71); -lean_inc(x_65); -x_73 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_chopUpChildren(x_65, x_69, x_72); +x_71 = lean_array_get_size(x_67); +x_72 = l_Array_toSubarray___redArg(x_67, x_70, x_71); +lean_inc(x_64); +x_73 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_chopUpChildren(x_64, x_69, x_72); lean_dec(x_69); x_74 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_74, 0, x_73); x_32 = x_64; -x_33 = x_63; -x_34 = x_65; +x_33 = x_65; +x_34 = x_68; x_35 = x_74; -x_36 = x_68; +x_36 = x_63; x_37 = lean_box(0); goto block_62; } @@ -13272,11 +13272,11 @@ lean_object* x_82; lean_object* x_83; x_82 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__0; x_83 = lean_ctor_get(x_82, 1); lean_inc(x_83); -x_63 = x_78; +x_63 = x_76; x_64 = x_77; -x_65 = x_76; -x_66 = x_79; -x_67 = lean_box(0); +x_65 = x_78; +x_66 = lean_box(0); +x_67 = x_80; x_68 = x_81; x_69 = x_83; goto block_75; @@ -13286,23 +13286,23 @@ goto block_75; size_t x_92; size_t x_93; lean_object* x_94; x_92 = lean_array_size(x_89); x_93 = 0; -x_94 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go_spec__1(x_88, x_1, x_92, x_93, x_89); -if (lean_obj_tag(x_88) == 0) +x_94 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go_spec__1(x_86, x_1, x_92, x_93, x_89); +if (lean_obj_tag(x_86) == 0) { x_76 = x_85; -x_77 = x_86; -x_78 = x_87; -x_79 = x_94; -x_80 = lean_box(0); +x_77 = x_87; +x_78 = x_88; +x_79 = lean_box(0); +x_80 = x_94; x_81 = x_91; goto block_84; } else { lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_95 = lean_ctor_get(x_88, 0); +x_95 = lean_ctor_get(x_86, 0); lean_inc(x_95); -lean_dec_ref(x_88); +lean_dec_ref(x_86); x_96 = lean_ctor_get(x_95, 3); lean_inc(x_96); lean_dec(x_95); @@ -13312,10 +13312,10 @@ lean_dec(x_96); if (lean_obj_tag(x_98) == 0) { x_76 = x_85; -x_77 = x_86; -x_78 = x_87; -x_79 = x_94; -x_80 = lean_box(0); +x_77 = x_87; +x_78 = x_88; +x_79 = lean_box(0); +x_80 = x_94; x_81 = x_91; goto block_84; } @@ -13325,11 +13325,11 @@ lean_object* x_99; x_99 = lean_ctor_get(x_98, 0); lean_inc(x_99); lean_dec_ref(x_98); -x_63 = x_87; -x_64 = x_86; -x_65 = x_85; -x_66 = x_94; -x_67 = lean_box(0); +x_63 = x_85; +x_64 = x_87; +x_65 = x_88; +x_66 = lean_box(0); +x_67 = x_94; x_68 = x_91; x_69 = x_99; goto block_75; @@ -13341,7 +13341,7 @@ goto block_75; size_t x_108; size_t x_109; lean_object* x_110; x_108 = lean_array_size(x_105); x_109 = 0; -x_110 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go_spec__0(x_1, x_104, x_108, x_109, x_105, x_107); +x_110 = l___private_Init_Data_Array_Basic_0__Array_mapMUnsafe_map___at___00__private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go_spec__0(x_1, x_102, x_108, x_109, x_105, x_101); if (lean_obj_tag(x_110) == 0) { lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; @@ -13356,8 +13356,8 @@ lean_dec(x_111); x_114 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_114, 0, x_112); x_32 = x_103; -x_33 = x_102; -x_34 = x_101; +x_33 = x_104; +x_34 = x_107; x_35 = x_114; x_36 = x_113; x_37 = lean_box(0); @@ -13366,8 +13366,8 @@ goto block_62; else { uint8_t x_115; -lean_dec(x_102); -lean_dec(x_101); +lean_dec(x_107); +lean_dec(x_103); x_115 = !lean_is_exclusive(x_110); if (x_115 == 0) { @@ -13387,54 +13387,54 @@ return x_117; } block_128: { -if (x_120 == 0) +if (x_122 == 0) { -x_101 = x_119; -x_102 = x_124; -x_103 = x_120; -x_104 = x_121; -x_105 = x_122; +x_101 = x_125; +x_102 = x_120; +x_103 = x_121; +x_104 = x_122; +x_105 = x_123; x_106 = lean_box(0); -x_107 = x_125; +x_107 = x_124; goto block_118; } else { uint8_t x_127; -x_127 = l_Array_isEmpty___redArg(x_122); +x_127 = l_Array_isEmpty___redArg(x_123); if (x_127 == 0) { -x_85 = x_119; +x_85 = x_125; x_86 = x_120; -x_87 = x_124; -x_88 = x_121; -x_89 = x_122; +x_87 = x_121; +x_88 = x_122; +x_89 = x_123; x_90 = lean_box(0); -x_91 = x_125; +x_91 = x_124; goto block_100; } else { -if (x_123 == 0) +if (x_119 == 0) { -x_101 = x_119; -x_102 = x_124; -x_103 = x_120; -x_104 = x_121; -x_105 = x_122; +x_101 = x_125; +x_102 = x_120; +x_103 = x_121; +x_104 = x_122; +x_105 = x_123; x_106 = lean_box(0); -x_107 = x_125; +x_107 = x_124; goto block_118; } else { -x_85 = x_119; +x_85 = x_125; x_86 = x_120; -x_87 = x_124; -x_88 = x_121; -x_89 = x_122; +x_87 = x_121; +x_88 = x_122; +x_89 = x_123; x_90 = lean_box(0); -x_91 = x_125; +x_91 = x_124; goto block_100; } } @@ -13444,7 +13444,7 @@ goto block_100; { lean_object* x_139; double x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; x_139 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__2; -x_140 = lean_float_sub(x_137, x_132); +x_140 = lean_float_sub(x_134, x_131); x_141 = lean_float_to_string(x_140); x_142 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_142, 0, x_141); @@ -13457,11 +13457,11 @@ lean_ctor_set(x_145, 0, x_143); lean_ctor_set(x_145, 1, x_144); x_146 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_146, 0, x_145); -lean_ctor_set(x_146, 1, x_134); +lean_ctor_set(x_146, 1, x_137); x_119 = x_130; x_120 = x_129; -x_121 = x_131; -x_122 = x_133; +x_121 = x_132; +x_122 = x_135; x_123 = x_136; x_124 = x_146; x_125 = x_138; @@ -13504,15 +13504,15 @@ x_165 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToIntera x_166 = lean_float_beq(x_155, x_165); if (x_166 == 0) { -x_129 = x_157; -x_130 = x_154; -x_131 = x_148; -x_132 = x_155; -x_133 = x_151; -x_134 = x_160; -x_135 = lean_box(0); -x_136 = x_158; -x_137 = x_156; +x_129 = x_148; +x_130 = x_158; +x_131 = x_155; +x_132 = x_154; +x_133 = lean_box(0); +x_134 = x_156; +x_135 = x_157; +x_136 = x_151; +x_137 = x_160; x_138 = x_163; goto block_147; } @@ -13520,11 +13520,11 @@ else { if (x_158 == 0) { -x_119 = x_154; -x_120 = x_157; -x_121 = x_148; -x_122 = x_151; -x_123 = x_158; +x_119 = x_158; +x_120 = x_148; +x_121 = x_154; +x_122 = x_157; +x_123 = x_151; x_124 = x_160; x_125 = x_163; x_126 = lean_box(0); @@ -13532,15 +13532,15 @@ goto block_128; } else { -x_129 = x_157; -x_130 = x_154; -x_131 = x_148; -x_132 = x_155; -x_133 = x_151; -x_134 = x_160; -x_135 = lean_box(0); -x_136 = x_158; -x_137 = x_156; +x_129 = x_148; +x_130 = x_158; +x_131 = x_155; +x_132 = x_154; +x_133 = lean_box(0); +x_134 = x_156; +x_135 = x_157; +x_136 = x_151; +x_137 = x_160; x_138 = x_163; goto block_147; } @@ -13562,15 +13562,15 @@ x_171 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToIntera x_172 = lean_float_beq(x_155, x_171); if (x_172 == 0) { -x_129 = x_157; -x_130 = x_154; -x_131 = x_148; -x_132 = x_155; -x_133 = x_151; -x_134 = x_170; -x_135 = lean_box(0); -x_136 = x_158; -x_137 = x_156; +x_129 = x_148; +x_130 = x_158; +x_131 = x_155; +x_132 = x_154; +x_133 = lean_box(0); +x_134 = x_156; +x_135 = x_157; +x_136 = x_151; +x_137 = x_170; x_138 = x_168; goto block_147; } @@ -13578,11 +13578,11 @@ else { if (x_158 == 0) { -x_119 = x_154; -x_120 = x_157; -x_121 = x_148; -x_122 = x_151; -x_123 = x_158; +x_119 = x_158; +x_120 = x_148; +x_121 = x_154; +x_122 = x_157; +x_123 = x_151; x_124 = x_170; x_125 = x_168; x_126 = lean_box(0); @@ -13590,15 +13590,15 @@ goto block_128; } else { -x_129 = x_157; -x_130 = x_154; -x_131 = x_148; -x_132 = x_155; -x_133 = x_151; -x_134 = x_170; -x_135 = lean_box(0); -x_136 = x_158; -x_137 = x_156; +x_129 = x_148; +x_130 = x_158; +x_131 = x_155; +x_132 = x_154; +x_133 = lean_box(0); +x_134 = x_156; +x_135 = x_157; +x_136 = x_151; +x_137 = x_170; x_138 = x_168; goto block_147; } @@ -14160,7 +14160,7 @@ return x_296; block_329: { lean_object* x_323; lean_object* x_324; -x_323 = lean_apply_2(x_319, x_322, lean_box(0)); +x_323 = lean_apply_2(x_321, x_322, lean_box(0)); x_324 = l___private_Init_Dynamic_0__Dynamic_get_x3fImpl___redArg(x_323, x_317); lean_dec(x_323); if (lean_obj_tag(x_324) == 1) @@ -14169,7 +14169,7 @@ lean_object* x_325; x_325 = lean_ctor_get(x_324, 0); lean_inc(x_325); lean_dec_ref(x_324); -x_2 = x_321; +x_2 = x_319; x_3 = x_325; x_4 = x_318; goto _start; @@ -14178,7 +14178,7 @@ else { lean_object* x_327; lean_object* x_328; lean_dec(x_324); -lean_dec(x_321); +lean_dec(x_319); lean_dec_ref(x_318); lean_dec_ref(x_1); x_327 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__8; @@ -15648,7 +15648,7 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractiveDiagnostic(lean_object* x_1, lean_object* x_2, uint8_t x_3) { _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_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_118; lean_object* x_119; lean_object* x_122; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_118; lean_object* x_119; lean_object* x_122; x_19 = lean_ctor_get(x_2, 1); lean_inc_ref(x_19); x_20 = lean_ctor_get(x_2, 2); @@ -15682,18 +15682,18 @@ goto block_141; { lean_object* x_15; lean_object* x_16; lean_object* x_17; x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_5); +lean_ctor_set(x_15, 0, x_11); x_16 = lean_box(0); x_17 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_15); -lean_ctor_set(x_17, 2, x_6); -lean_ctor_set(x_17, 3, x_11); +lean_ctor_set(x_17, 2, x_5); +lean_ctor_set(x_17, 3, x_13); lean_ctor_set(x_17, 4, x_14); -lean_ctor_set(x_17, 5, x_12); -lean_ctor_set(x_17, 6, x_13); -lean_ctor_set(x_17, 7, x_10); -lean_ctor_set(x_17, 8, x_9); +lean_ctor_set(x_17, 5, x_6); +lean_ctor_set(x_17, 6, x_9); +lean_ctor_set(x_17, 7, x_7); +lean_ctor_set(x_17, 8, x_12); lean_ctor_set(x_17, 9, x_16); lean_ctor_set(x_17, 10, x_16); return x_17; @@ -15710,14 +15710,14 @@ if (lean_obj_tag(x_36) == 0) lean_object* x_37; x_37 = lean_box(0); x_5 = x_25; -x_6 = x_27; -x_7 = x_26; -x_8 = lean_box(0); -x_9 = x_28; -x_10 = x_30; -x_11 = x_32; +x_6 = x_26; +x_7 = x_28; +x_8 = x_27; +x_9 = x_34; +x_10 = lean_box(0); +x_11 = x_29; x_12 = x_33; -x_13 = x_34; +x_13 = x_32; x_14 = x_37; goto block_18; } @@ -15734,14 +15734,14 @@ x_41 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_36, 0, x_41); x_5 = x_25; -x_6 = x_27; -x_7 = x_26; -x_8 = lean_box(0); -x_9 = x_28; -x_10 = x_30; -x_11 = x_32; +x_6 = x_26; +x_7 = x_28; +x_8 = x_27; +x_9 = x_34; +x_10 = lean_box(0); +x_11 = x_29; x_12 = x_33; -x_13 = x_34; +x_13 = x_32; x_14 = x_36; goto block_18; } @@ -15757,14 +15757,14 @@ lean_ctor_set(x_44, 0, x_43); x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_44); x_5 = x_25; -x_6 = x_27; -x_7 = x_26; -x_8 = lean_box(0); -x_9 = x_28; -x_10 = x_30; -x_11 = x_32; +x_6 = x_26; +x_7 = x_28; +x_8 = x_27; +x_9 = x_34; +x_10 = lean_box(0); +x_11 = x_29; x_12 = x_33; -x_13 = x_34; +x_13 = x_32; x_14 = x_45; goto block_18; } @@ -15785,12 +15785,12 @@ lean_dec_ref(x_56); x_25 = x_47; x_26 = x_48; x_27 = x_49; -x_28 = x_54; -x_29 = lean_box(0); -x_30 = x_50; -x_31 = x_51; -x_32 = x_52; -x_33 = x_53; +x_28 = x_50; +x_29 = x_51; +x_30 = lean_box(0); +x_31 = x_52; +x_32 = x_53; +x_33 = x_54; x_34 = x_57; goto block_46; } @@ -15813,12 +15813,12 @@ lean_ctor_set(x_56, 0, x_64); x_25 = x_47; x_26 = x_48; x_27 = x_49; -x_28 = x_54; -x_29 = lean_box(0); -x_30 = x_50; -x_31 = x_51; -x_32 = x_52; -x_33 = x_53; +x_28 = x_50; +x_29 = x_51; +x_30 = lean_box(0); +x_31 = x_52; +x_32 = x_53; +x_33 = x_54; x_34 = x_56; goto block_46; } @@ -15839,12 +15839,12 @@ lean_ctor_set(x_71, 0, x_70); x_25 = x_47; x_26 = x_48; x_27 = x_49; -x_28 = x_54; -x_29 = lean_box(0); -x_30 = x_50; -x_31 = x_51; -x_32 = x_52; -x_33 = x_53; +x_28 = x_50; +x_29 = x_51; +x_30 = lean_box(0); +x_31 = x_52; +x_32 = x_53; +x_33 = x_54; x_34 = x_71; goto block_46; } @@ -15865,11 +15865,11 @@ if (x_83 == 0) lean_object* x_84; x_84 = lean_box(0); x_47 = x_75; -x_48 = x_77; -x_49 = x_76; +x_48 = x_76; +x_49 = x_77; x_50 = x_81; -x_51 = x_79; -x_52 = x_78; +x_51 = x_78; +x_52 = x_79; x_53 = x_80; x_54 = x_84; goto block_72; @@ -15879,11 +15879,11 @@ else lean_object* x_85; x_85 = l_Lean_Widget_msgToInteractiveDiagnostic___closed__4; x_47 = x_75; -x_48 = x_77; -x_49 = x_76; +x_48 = x_76; +x_49 = x_77; x_50 = x_81; -x_51 = x_79; -x_52 = x_78; +x_51 = x_78; +x_52 = x_79; x_53 = x_80; x_54 = x_85; goto block_72; @@ -15895,11 +15895,11 @@ lean_object* x_86; lean_dec_ref(x_73); x_86 = l_Lean_Widget_msgToInteractiveDiagnostic___closed__6; x_47 = x_75; -x_48 = x_77; -x_49 = x_76; +x_48 = x_76; +x_49 = x_77; x_50 = x_81; -x_51 = x_79; -x_52 = x_78; +x_51 = x_78; +x_52 = x_79; x_53 = x_80; x_54 = x_86; goto block_72; @@ -15921,11 +15921,11 @@ if (x_95 == 0) lean_object* x_96; x_96 = lean_box(0); x_75 = x_88; -x_76 = x_90; +x_76 = x_93; x_77 = x_89; -x_78 = x_92; +x_78 = x_90; x_79 = x_91; -x_80 = x_93; +x_80 = x_92; x_81 = x_96; goto block_87; } @@ -15934,11 +15934,11 @@ else lean_object* x_97; x_97 = l_Lean_Widget_msgToInteractiveDiagnostic___closed__11; x_75 = x_88; -x_76 = x_90; +x_76 = x_93; x_77 = x_89; -x_78 = x_92; +x_78 = x_90; x_79 = x_91; -x_80 = x_93; +x_80 = x_92; x_81 = x_97; goto block_87; } @@ -15948,11 +15948,11 @@ else lean_object* x_98; x_98 = l_Lean_Widget_msgToInteractiveDiagnostic___closed__13; x_75 = x_88; -x_76 = x_90; +x_76 = x_93; x_77 = x_89; -x_78 = x_92; +x_78 = x_90; x_79 = x_91; -x_80 = x_93; +x_80 = x_92; x_81 = x_98; goto block_87; } @@ -15968,9 +15968,9 @@ if (x_23 == 0) { lean_object* x_106; x_106 = lean_box(0); -x_88 = x_100; -x_89 = x_101; -x_90 = x_104; +x_88 = x_104; +x_89 = x_100; +x_90 = x_101; x_91 = x_105; x_92 = x_106; goto block_99; @@ -15979,9 +15979,9 @@ else { lean_object* x_107; x_107 = l_Lean_Widget_msgToInteractiveDiagnostic___closed__14; -x_88 = x_100; -x_89 = x_101; -x_90 = x_104; +x_88 = x_104; +x_89 = x_100; +x_90 = x_101; x_91 = x_105; x_92 = x_107; goto block_99; @@ -16002,8 +16002,8 @@ case 0: { uint8_t x_114; x_114 = 2; -x_100 = x_113; -x_101 = x_112; +x_100 = x_112; +x_101 = x_113; x_102 = x_114; goto block_108; } @@ -16011,8 +16011,8 @@ case 1: { uint8_t x_115; x_115 = 1; -x_100 = x_113; -x_101 = x_112; +x_100 = x_112; +x_101 = x_113; x_102 = x_115; goto block_108; } @@ -16020,8 +16020,8 @@ goto block_108; { uint8_t x_116; x_116 = 0; -x_100 = x_113; -x_101 = x_112; +x_100 = x_112; +x_101 = x_113; x_102 = x_116; goto block_108; } diff --git a/stage0/stdlib/Std/Data/DTreeMap/Internal/Balancing.c b/stage0/stdlib/Std/Data/DTreeMap/Internal/Balancing.c index 018d5825f2e0..7b36ed05b7cc 100644 --- a/stage0/stdlib/Std/Data/DTreeMap/Internal/Balancing.c +++ b/stage0/stdlib/Std/Data/DTreeMap/Internal/Balancing.c @@ -1737,9 +1737,9 @@ goto block_51; block_43: { lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_nat_add(x_38, x_39); +x_40 = lean_nat_add(x_37, x_39); lean_dec(x_39); -lean_dec(x_38); +lean_dec(x_37); if (lean_is_scalar(x_33)) { x_41 = lean_alloc_ctor(0, 5, 0); } else { @@ -1758,7 +1758,7 @@ if (lean_is_scalar(x_23)) { lean_ctor_set(x_42, 0, x_36); lean_ctor_set(x_42, 1, x_26); lean_ctor_set(x_42, 2, x_27); -lean_ctor_set(x_42, 3, x_37); +lean_ctor_set(x_42, 3, x_38); lean_ctor_set(x_42, 4, x_41); return x_42; } @@ -1780,8 +1780,8 @@ if (lean_obj_tag(x_29) == 0) lean_object* x_49; x_49 = lean_ctor_get(x_29, 0); lean_inc(x_49); -x_37 = x_47; -x_38 = x_48; +x_37 = x_48; +x_38 = x_47; x_39 = x_49; goto block_43; } @@ -1789,8 +1789,8 @@ else { lean_object* x_50; x_50 = lean_unsigned_to_nat(0u); -x_37 = x_47; -x_38 = x_48; +x_37 = x_48; +x_38 = x_47; x_39 = x_50; goto block_43; } @@ -2198,9 +2198,9 @@ goto block_46; block_38: { lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_nat_add(x_33, x_34); +x_35 = lean_nat_add(x_32, x_34); lean_dec(x_34); -lean_dec(x_33); +lean_dec(x_32); if (lean_is_scalar(x_28)) { x_36 = lean_alloc_ctor(0, 5, 0); } else { @@ -2219,7 +2219,7 @@ if (lean_is_scalar(x_18)) { lean_ctor_set(x_37, 0, x_31); lean_ctor_set(x_37, 1, x_21); lean_ctor_set(x_37, 2, x_22); -lean_ctor_set(x_37, 3, x_32); +lean_ctor_set(x_37, 3, x_33); lean_ctor_set(x_37, 4, x_36); return x_37; } @@ -2241,8 +2241,8 @@ if (lean_obj_tag(x_24) == 0) lean_object* x_44; x_44 = lean_ctor_get(x_24, 0); lean_inc(x_44); -x_32 = x_42; -x_33 = x_43; +x_32 = x_43; +x_33 = x_42; x_34 = x_44; goto block_38; } @@ -2250,8 +2250,8 @@ else { lean_object* x_45; x_45 = lean_unsigned_to_nat(0u); -x_32 = x_42; -x_33 = x_43; +x_32 = x_43; +x_33 = x_42; x_34 = x_45; goto block_38; } @@ -2659,9 +2659,9 @@ goto block_51; block_43: { lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_nat_add(x_38, x_39); +x_40 = lean_nat_add(x_37, x_39); lean_dec(x_39); -lean_dec(x_38); +lean_dec(x_37); if (lean_is_scalar(x_33)) { x_41 = lean_alloc_ctor(0, 5, 0); } else { @@ -2680,7 +2680,7 @@ if (lean_is_scalar(x_23)) { lean_ctor_set(x_42, 0, x_36); lean_ctor_set(x_42, 1, x_26); lean_ctor_set(x_42, 2, x_27); -lean_ctor_set(x_42, 3, x_37); +lean_ctor_set(x_42, 3, x_38); lean_ctor_set(x_42, 4, x_41); return x_42; } @@ -2702,8 +2702,8 @@ if (lean_obj_tag(x_29) == 0) lean_object* x_49; x_49 = lean_ctor_get(x_29, 0); lean_inc(x_49); -x_37 = x_47; -x_38 = x_48; +x_37 = x_48; +x_38 = x_47; x_39 = x_49; goto block_43; } @@ -2711,8 +2711,8 @@ else { lean_object* x_50; x_50 = lean_unsigned_to_nat(0u); -x_37 = x_47; -x_38 = x_48; +x_37 = x_48; +x_38 = x_47; x_39 = x_50; goto block_43; } @@ -3228,9 +3228,9 @@ goto block_46; block_38: { lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_nat_add(x_33, x_34); +x_35 = lean_nat_add(x_32, x_34); lean_dec(x_34); -lean_dec(x_33); +lean_dec(x_32); if (lean_is_scalar(x_28)) { x_36 = lean_alloc_ctor(0, 5, 0); } else { @@ -3249,7 +3249,7 @@ if (lean_is_scalar(x_18)) { lean_ctor_set(x_37, 0, x_31); lean_ctor_set(x_37, 1, x_21); lean_ctor_set(x_37, 2, x_22); -lean_ctor_set(x_37, 3, x_32); +lean_ctor_set(x_37, 3, x_33); lean_ctor_set(x_37, 4, x_36); return x_37; } @@ -3271,8 +3271,8 @@ if (lean_obj_tag(x_24) == 0) lean_object* x_44; x_44 = lean_ctor_get(x_24, 0); lean_inc(x_44); -x_32 = x_42; -x_33 = x_43; +x_32 = x_43; +x_33 = x_42; x_34 = x_44; goto block_38; } @@ -3280,8 +3280,8 @@ else { lean_object* x_45; x_45 = lean_unsigned_to_nat(0u); -x_32 = x_42; -x_33 = x_43; +x_32 = x_43; +x_33 = x_42; x_34 = x_45; goto block_38; } @@ -3852,9 +3852,9 @@ goto block_48; block_40: { lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_nat_add(x_34, x_36); +x_37 = lean_nat_add(x_35, x_36); lean_dec(x_36); -lean_dec(x_34); +lean_dec(x_35); if (lean_is_scalar(x_30)) { x_38 = lean_alloc_ctor(0, 5, 0); } else { @@ -3873,7 +3873,7 @@ if (lean_is_scalar(x_20)) { lean_ctor_set(x_39, 0, x_33); lean_ctor_set(x_39, 1, x_23); lean_ctor_set(x_39, 2, x_24); -lean_ctor_set(x_39, 3, x_35); +lean_ctor_set(x_39, 3, x_34); lean_ctor_set(x_39, 4, x_38); return x_39; } @@ -3895,8 +3895,8 @@ if (lean_obj_tag(x_26) == 0) lean_object* x_46; x_46 = lean_ctor_get(x_26, 0); lean_inc(x_46); -x_34 = x_45; -x_35 = x_44; +x_34 = x_44; +x_35 = x_45; x_36 = x_46; goto block_40; } @@ -3904,8 +3904,8 @@ else { lean_object* x_47; x_47 = lean_unsigned_to_nat(0u); -x_34 = x_45; -x_35 = x_44; +x_34 = x_44; +x_35 = x_45; x_36 = x_47; goto block_40; } @@ -4460,9 +4460,9 @@ goto block_46; block_38: { lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_nat_add(x_32, x_34); +x_35 = lean_nat_add(x_33, x_34); lean_dec(x_34); -lean_dec(x_32); +lean_dec(x_33); if (lean_is_scalar(x_28)) { x_36 = lean_alloc_ctor(0, 5, 0); } else { @@ -4481,7 +4481,7 @@ if (lean_is_scalar(x_18)) { lean_ctor_set(x_37, 0, x_31); lean_ctor_set(x_37, 1, x_21); lean_ctor_set(x_37, 2, x_22); -lean_ctor_set(x_37, 3, x_33); +lean_ctor_set(x_37, 3, x_32); lean_ctor_set(x_37, 4, x_36); return x_37; } @@ -4503,8 +4503,8 @@ if (lean_obj_tag(x_24) == 0) lean_object* x_44; x_44 = lean_ctor_get(x_24, 0); lean_inc(x_44); -x_32 = x_43; -x_33 = x_42; +x_32 = x_42; +x_33 = x_43; x_34 = x_44; goto block_38; } @@ -4512,8 +4512,8 @@ else { lean_object* x_45; x_45 = lean_unsigned_to_nat(0u); -x_32 = x_43; -x_33 = x_42; +x_32 = x_42; +x_33 = x_43; x_34 = x_45; goto block_38; } @@ -8233,9 +8233,9 @@ goto block_58; block_50: { lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_nat_add(x_38, x_40); +x_41 = lean_nat_add(x_39, x_40); lean_dec(x_40); -lean_dec(x_38); +lean_dec(x_39); lean_inc_ref(x_4); if (lean_is_scalar(x_34)) { x_42 = lean_alloc_ctor(0, 5, 0); @@ -8262,7 +8262,7 @@ lean_dec(x_47); x_48 = lean_ctor_get(x_4, 0); lean_dec(x_48); lean_ctor_set(x_4, 4, x_42); -lean_ctor_set(x_4, 3, x_39); +lean_ctor_set(x_4, 3, x_38); lean_ctor_set(x_4, 2, x_28); lean_ctor_set(x_4, 1, x_27); lean_ctor_set(x_4, 0, x_37); @@ -8276,7 +8276,7 @@ x_49 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_49, 0, x_37); lean_ctor_set(x_49, 1, x_27); lean_ctor_set(x_49, 2, x_28); -lean_ctor_set(x_49, 3, x_39); +lean_ctor_set(x_49, 3, x_38); lean_ctor_set(x_49, 4, x_42); return x_49; } @@ -8303,8 +8303,8 @@ if (lean_obj_tag(x_30) == 0) lean_object* x_56; x_56 = lean_ctor_get(x_30, 0); lean_inc(x_56); -x_38 = x_55; -x_39 = x_54; +x_38 = x_54; +x_39 = x_55; x_40 = x_56; goto block_50; } @@ -8312,8 +8312,8 @@ else { lean_object* x_57; x_57 = lean_unsigned_to_nat(0u); -x_38 = x_55; -x_39 = x_54; +x_38 = x_54; +x_39 = x_55; x_40 = x_57; goto block_50; } @@ -9339,9 +9339,9 @@ goto block_58; block_50: { lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_nat_add(x_39, x_40); +x_41 = lean_nat_add(x_38, x_40); lean_dec(x_40); -lean_dec(x_39); +lean_dec(x_38); lean_inc_ref(x_4); if (lean_is_scalar(x_34)) { x_42 = lean_alloc_ctor(0, 5, 0); @@ -9368,7 +9368,7 @@ lean_dec(x_47); x_48 = lean_ctor_get(x_4, 0); lean_dec(x_48); lean_ctor_set(x_4, 4, x_42); -lean_ctor_set(x_4, 3, x_38); +lean_ctor_set(x_4, 3, x_39); lean_ctor_set(x_4, 2, x_28); lean_ctor_set(x_4, 1, x_27); lean_ctor_set(x_4, 0, x_37); @@ -9382,7 +9382,7 @@ x_49 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_49, 0, x_37); lean_ctor_set(x_49, 1, x_27); lean_ctor_set(x_49, 2, x_28); -lean_ctor_set(x_49, 3, x_38); +lean_ctor_set(x_49, 3, x_39); lean_ctor_set(x_49, 4, x_42); return x_49; } @@ -9409,8 +9409,8 @@ if (lean_obj_tag(x_30) == 0) lean_object* x_56; x_56 = lean_ctor_get(x_30, 0); lean_inc(x_56); -x_38 = x_54; -x_39 = x_55; +x_38 = x_55; +x_39 = x_54; x_40 = x_56; goto block_50; } @@ -9418,8 +9418,8 @@ else { lean_object* x_57; x_57 = lean_unsigned_to_nat(0u); -x_38 = x_54; -x_39 = x_55; +x_38 = x_55; +x_39 = x_54; x_40 = x_57; goto block_50; } @@ -9562,9 +9562,9 @@ goto block_99; block_92: { lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_nat_add(x_87, x_88); +x_89 = lean_nat_add(x_86, x_88); lean_dec(x_88); -lean_dec(x_87); +lean_dec(x_86); if (lean_is_scalar(x_82)) { x_90 = lean_alloc_ctor(0, 5, 0); } else { @@ -9583,7 +9583,7 @@ if (lean_is_scalar(x_72)) { lean_ctor_set(x_91, 0, x_85); lean_ctor_set(x_91, 1, x_74); lean_ctor_set(x_91, 2, x_75); -lean_ctor_set(x_91, 3, x_86); +lean_ctor_set(x_91, 3, x_87); lean_ctor_set(x_91, 4, x_90); return x_91; } @@ -9605,8 +9605,8 @@ if (lean_obj_tag(x_77) == 0) lean_object* x_97; x_97 = lean_ctor_get(x_77, 0); lean_inc(x_97); -x_86 = x_95; -x_87 = x_96; +x_86 = x_96; +x_87 = x_95; x_88 = x_97; goto block_92; } @@ -9614,8 +9614,8 @@ else { lean_object* x_98; x_98 = lean_unsigned_to_nat(0u); -x_86 = x_95; -x_87 = x_96; +x_86 = x_96; +x_87 = x_95; x_88 = x_98; goto block_92; } @@ -10613,11 +10613,11 @@ goto block_25; block_20: { lean_object* x_11; uint8_t x_12; -x_11 = lean_nat_mul(x_9, x_10); +x_11 = lean_nat_mul(x_8, x_10); lean_dec(x_10); -x_12 = lean_nat_dec_lt(x_8, x_11); +x_12 = lean_nat_dec_lt(x_9, x_11); lean_dec(x_11); -lean_dec(x_8); +lean_dec(x_9); if (x_12 == 0) { if (lean_obj_tag(x_6) == 0) @@ -10658,8 +10658,8 @@ if (lean_obj_tag(x_5) == 0) lean_object* x_23; x_23 = lean_ctor_get(x_5, 0); lean_inc(x_23); -x_8 = x_21; -x_9 = x_22; +x_8 = x_22; +x_9 = x_21; x_10 = x_23; goto block_20; } @@ -10667,8 +10667,8 @@ else { lean_object* x_24; x_24 = lean_unsigned_to_nat(0u); -x_8 = x_21; -x_9 = x_22; +x_8 = x_22; +x_9 = x_21; x_10 = x_24; goto block_20; } diff --git a/stage0/stdlib/Std/Data/DTreeMap/Internal/Operations.c b/stage0/stdlib/Std/Data/DTreeMap/Internal/Operations.c index 1b366205061a..559c9b092b53 100644 --- a/stage0/stdlib/Std/Data/DTreeMap/Internal/Operations.c +++ b/stage0/stdlib/Std/Data/DTreeMap/Internal/Operations.c @@ -435,17 +435,17 @@ if (lean_obj_tag(x_71) == 0) lean_object* x_80; x_80 = lean_ctor_get(x_71, 0); lean_inc(x_80); -x_30 = x_50; -x_31 = x_78; -x_32 = x_73; -x_33 = x_53; -x_34 = x_72; -x_35 = x_71; -x_36 = x_77; -x_37 = x_51; -x_38 = x_79; -x_39 = x_70; -x_40 = x_69; +x_30 = x_69; +x_31 = x_77; +x_32 = x_72; +x_33 = x_51; +x_34 = x_53; +x_35 = x_73; +x_36 = x_71; +x_37 = x_50; +x_38 = x_70; +x_39 = x_79; +x_40 = x_78; x_41 = x_80; goto block_47; } @@ -453,17 +453,17 @@ else { lean_object* x_81; x_81 = lean_unsigned_to_nat(0u); -x_30 = x_50; -x_31 = x_78; -x_32 = x_73; -x_33 = x_53; -x_34 = x_72; -x_35 = x_71; -x_36 = x_77; -x_37 = x_51; -x_38 = x_79; -x_39 = x_70; -x_40 = x_69; +x_30 = x_69; +x_31 = x_77; +x_32 = x_72; +x_33 = x_51; +x_34 = x_53; +x_35 = x_73; +x_36 = x_71; +x_37 = x_50; +x_38 = x_70; +x_39 = x_79; +x_40 = x_78; x_41 = x_81; goto block_47; } @@ -560,17 +560,17 @@ if (lean_obj_tag(x_98) == 0) lean_object* x_107; x_107 = lean_ctor_get(x_98, 0); lean_inc(x_107); -x_30 = x_50; -x_31 = x_105; -x_32 = x_100; -x_33 = x_53; -x_34 = x_99; -x_35 = x_98; -x_36 = x_104; -x_37 = x_51; -x_38 = x_106; -x_39 = x_97; -x_40 = x_96; +x_30 = x_96; +x_31 = x_104; +x_32 = x_99; +x_33 = x_51; +x_34 = x_53; +x_35 = x_100; +x_36 = x_98; +x_37 = x_50; +x_38 = x_97; +x_39 = x_106; +x_40 = x_105; x_41 = x_107; goto block_47; } @@ -578,17 +578,17 @@ else { lean_object* x_108; x_108 = lean_unsigned_to_nat(0u); -x_30 = x_50; -x_31 = x_105; -x_32 = x_100; -x_33 = x_53; -x_34 = x_99; -x_35 = x_98; -x_36 = x_104; -x_37 = x_51; -x_38 = x_106; -x_39 = x_97; -x_40 = x_96; +x_30 = x_96; +x_31 = x_104; +x_32 = x_99; +x_33 = x_51; +x_34 = x_53; +x_35 = x_100; +x_36 = x_98; +x_37 = x_50; +x_38 = x_97; +x_39 = x_106; +x_40 = x_105; x_41 = x_108; goto block_47; } @@ -1022,22 +1022,22 @@ return x_211; block_29: { lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_nat_add(x_18, x_24); +x_25 = lean_nat_add(x_20, x_24); lean_dec(x_24); -lean_dec(x_18); +lean_dec(x_20); if (lean_is_scalar(x_9)) { x_26 = lean_alloc_ctor(0, 5, 0); } else { x_26 = x_9; } lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_15); -lean_ctor_set(x_26, 2, x_21); -lean_ctor_set(x_26, 3, x_19); -lean_ctor_set(x_26, 4, x_17); +lean_ctor_set(x_26, 1, x_21); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_17); +lean_ctor_set(x_26, 4, x_18); x_27 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_27, 0, x_20); -lean_ctor_set(x_27, 1, x_23); +lean_ctor_set(x_27, 0, x_23); +lean_ctor_set(x_27, 1, x_15); lean_ctor_set(x_27, 2, x_22); lean_ctor_set(x_27, 3, x_16); lean_ctor_set(x_27, 4, x_26); @@ -1054,31 +1054,31 @@ return x_28; block_47: { lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_nat_add(x_31, x_41); +x_42 = lean_nat_add(x_40, x_41); lean_dec(x_41); -lean_dec(x_31); +lean_dec(x_40); x_43 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_1); lean_ctor_set(x_43, 2, x_2); lean_ctor_set(x_43, 3, x_13); -lean_ctor_set(x_43, 4, x_35); -x_44 = lean_nat_add(x_36, x_32); -lean_dec(x_32); -if (lean_obj_tag(x_34) == 0) +lean_ctor_set(x_43, 4, x_36); +x_44 = lean_nat_add(x_31, x_35); +lean_dec(x_35); +if (lean_obj_tag(x_32) == 0) { lean_object* x_45; -x_45 = lean_ctor_get(x_34, 0); +x_45 = lean_ctor_get(x_32, 0); lean_inc(x_45); x_15 = x_30; x_16 = x_43; -x_17 = x_33; -x_18 = x_44; -x_19 = x_34; -x_20 = x_38; +x_17 = x_32; +x_18 = x_34; +x_19 = x_33; +x_20 = x_44; x_21 = x_37; -x_22 = x_39; -x_23 = x_40; +x_22 = x_38; +x_23 = x_39; x_24 = x_45; goto block_29; } @@ -1088,13 +1088,13 @@ lean_object* x_46; x_46 = lean_unsigned_to_nat(0u); x_15 = x_30; x_16 = x_43; -x_17 = x_33; -x_18 = x_44; -x_19 = x_34; -x_20 = x_38; +x_17 = x_32; +x_18 = x_34; +x_19 = x_33; +x_20 = x_44; x_21 = x_37; -x_22 = x_39; -x_23 = x_40; +x_22 = x_38; +x_23 = x_39; x_24 = x_46; goto block_29; } @@ -2335,17 +2335,17 @@ lean_object* x_78; x_78 = lean_ctor_get(x_69, 0); lean_inc(x_78); lean_inc(x_45); -x_27 = x_77; -x_28 = x_76; -x_29 = x_70; -x_30 = x_45; -x_31 = x_67; -x_32 = x_47; -x_33 = x_69; -x_34 = x_48; -x_35 = x_74; -x_36 = x_49; -x_37 = x_68; +x_27 = x_70; +x_28 = x_77; +x_29 = x_45; +x_30 = x_48; +x_31 = x_68; +x_32 = x_69; +x_33 = x_47; +x_34 = x_74; +x_35 = x_49; +x_36 = x_76; +x_37 = x_67; x_38 = x_78; goto block_44; } @@ -2354,17 +2354,17 @@ else lean_object* x_79; x_79 = lean_unsigned_to_nat(0u); lean_inc(x_45); -x_27 = x_77; -x_28 = x_76; -x_29 = x_70; -x_30 = x_45; -x_31 = x_67; -x_32 = x_47; -x_33 = x_69; -x_34 = x_48; -x_35 = x_74; -x_36 = x_49; -x_37 = x_68; +x_27 = x_70; +x_28 = x_77; +x_29 = x_45; +x_30 = x_48; +x_31 = x_68; +x_32 = x_69; +x_33 = x_47; +x_34 = x_74; +x_35 = x_49; +x_36 = x_76; +x_37 = x_67; x_38 = x_79; goto block_44; } @@ -2465,17 +2465,17 @@ lean_object* x_107; x_107 = lean_ctor_get(x_98, 0); lean_inc(x_107); lean_inc(x_45); -x_27 = x_106; -x_28 = x_105; -x_29 = x_99; -x_30 = x_45; -x_31 = x_96; -x_32 = x_47; -x_33 = x_98; -x_34 = x_48; -x_35 = x_103; -x_36 = x_49; -x_37 = x_97; +x_27 = x_99; +x_28 = x_106; +x_29 = x_45; +x_30 = x_48; +x_31 = x_97; +x_32 = x_98; +x_33 = x_47; +x_34 = x_103; +x_35 = x_49; +x_36 = x_105; +x_37 = x_96; x_38 = x_107; goto block_44; } @@ -2484,17 +2484,17 @@ else lean_object* x_108; x_108 = lean_unsigned_to_nat(0u); lean_inc(x_45); -x_27 = x_106; -x_28 = x_105; -x_29 = x_99; -x_30 = x_45; -x_31 = x_96; -x_32 = x_47; -x_33 = x_98; -x_34 = x_48; -x_35 = x_103; -x_36 = x_49; -x_37 = x_97; +x_27 = x_99; +x_28 = x_106; +x_29 = x_45; +x_30 = x_48; +x_31 = x_97; +x_32 = x_98; +x_33 = x_47; +x_34 = x_103; +x_35 = x_49; +x_36 = x_105; +x_37 = x_96; x_38 = x_108; goto block_44; } @@ -2945,9 +2945,9 @@ return x_212; block_26: { lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_nat_add(x_17, x_21); +x_22 = lean_nat_add(x_20, x_21); lean_dec(x_21); -lean_dec(x_17); +lean_dec(x_20); if (lean_is_scalar(x_9)) { x_23 = lean_alloc_ctor(0, 5, 0); } else { @@ -2956,13 +2956,13 @@ if (lean_is_scalar(x_9)) { lean_ctor_set(x_23, 0, x_22); lean_ctor_set(x_23, 1, x_1); lean_ctor_set(x_23, 2, x_2); -lean_ctor_set(x_23, 3, x_16); +lean_ctor_set(x_23, 3, x_15); lean_ctor_set(x_23, 4, x_13); x_24 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_24, 0, x_15); -lean_ctor_set(x_24, 1, x_18); -lean_ctor_set(x_24, 2, x_20); -lean_ctor_set(x_24, 3, x_19); +lean_ctor_set(x_24, 0, x_18); +lean_ctor_set(x_24, 1, x_19); +lean_ctor_set(x_24, 2, x_17); +lean_ctor_set(x_24, 3, x_16); lean_ctor_set(x_24, 4, x_23); if (lean_is_scalar(x_14)) { x_25 = lean_alloc_ctor(0, 3, 0); @@ -2977,28 +2977,28 @@ return x_25; block_44: { lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_nat_add(x_27, x_38); +x_39 = lean_nat_add(x_28, x_38); lean_dec(x_38); -lean_dec(x_27); +lean_dec(x_28); x_40 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_32); -lean_ctor_set(x_40, 2, x_34); -lean_ctor_set(x_40, 3, x_36); -lean_ctor_set(x_40, 4, x_33); -x_41 = lean_nat_add(x_35, x_30); -lean_dec(x_30); -if (lean_obj_tag(x_29) == 0) +lean_ctor_set(x_40, 1, x_33); +lean_ctor_set(x_40, 2, x_30); +lean_ctor_set(x_40, 3, x_35); +lean_ctor_set(x_40, 4, x_32); +x_41 = lean_nat_add(x_34, x_29); +lean_dec(x_29); +if (lean_obj_tag(x_27) == 0) { lean_object* x_42; -x_42 = lean_ctor_get(x_29, 0); +x_42 = lean_ctor_get(x_27, 0); lean_inc(x_42); -x_15 = x_28; -x_16 = x_29; -x_17 = x_41; -x_18 = x_31; -x_19 = x_40; -x_20 = x_37; +x_15 = x_27; +x_16 = x_40; +x_17 = x_31; +x_18 = x_36; +x_19 = x_37; +x_20 = x_41; x_21 = x_42; goto block_26; } @@ -3006,12 +3006,12 @@ else { lean_object* x_43; x_43 = lean_unsigned_to_nat(0u); -x_15 = x_28; -x_16 = x_29; -x_17 = x_41; -x_18 = x_31; -x_19 = x_40; -x_20 = x_37; +x_15 = x_27; +x_16 = x_40; +x_17 = x_31; +x_18 = x_36; +x_19 = x_37; +x_20 = x_41; x_21 = x_43; goto block_26; } @@ -3238,9 +3238,9 @@ goto block_58; block_50: { lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_nat_add(x_44, x_45); +x_46 = lean_nat_add(x_43, x_45); lean_dec(x_45); -lean_dec(x_44); +lean_dec(x_43); if (lean_is_scalar(x_39)) { x_47 = lean_alloc_ctor(0, 5, 0); } else { @@ -3259,7 +3259,7 @@ if (lean_is_scalar(x_29)) { lean_ctor_set(x_48, 0, x_42); lean_ctor_set(x_48, 1, x_32); lean_ctor_set(x_48, 2, x_33); -lean_ctor_set(x_48, 3, x_43); +lean_ctor_set(x_48, 3, x_44); lean_ctor_set(x_48, 4, x_47); if (lean_is_scalar(x_14)) { x_49 = lean_alloc_ctor(0, 3, 0); @@ -3293,8 +3293,8 @@ if (lean_obj_tag(x_35) == 0) lean_object* x_56; x_56 = lean_ctor_get(x_35, 0); lean_inc(x_56); -x_43 = x_54; -x_44 = x_55; +x_43 = x_55; +x_44 = x_54; x_45 = x_56; goto block_50; } @@ -3302,8 +3302,8 @@ else { lean_object* x_57; x_57 = lean_unsigned_to_nat(0u); -x_43 = x_54; -x_44 = x_55; +x_43 = x_55; +x_44 = x_54; x_45 = x_57; goto block_50; } @@ -10261,9 +10261,9 @@ goto block_51; block_43: { lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_nat_add(x_37, x_39); +x_40 = lean_nat_add(x_38, x_39); lean_dec(x_39); -lean_dec(x_37); +lean_dec(x_38); if (lean_is_scalar(x_33)) { x_41 = lean_alloc_ctor(0, 5, 0); } else { @@ -10282,7 +10282,7 @@ if (lean_is_scalar(x_23)) { lean_ctor_set(x_42, 0, x_36); lean_ctor_set(x_42, 1, x_26); lean_ctor_set(x_42, 2, x_27); -lean_ctor_set(x_42, 3, x_38); +lean_ctor_set(x_42, 3, x_37); lean_ctor_set(x_42, 4, x_41); return x_42; } @@ -10308,8 +10308,8 @@ if (lean_obj_tag(x_29) == 0) lean_object* x_49; x_49 = lean_ctor_get(x_29, 0); lean_inc(x_49); -x_37 = x_48; -x_38 = x_47; +x_37 = x_47; +x_38 = x_48; x_39 = x_49; goto block_43; } @@ -10317,8 +10317,8 @@ else { lean_object* x_50; x_50 = lean_unsigned_to_nat(0u); -x_37 = x_48; -x_38 = x_47; +x_37 = x_47; +x_38 = x_48; x_39 = x_50; goto block_43; } @@ -10912,9 +10912,9 @@ goto block_49; block_42: { lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_nat_add(x_37, x_38); +x_39 = lean_nat_add(x_36, x_38); lean_dec(x_38); -lean_dec(x_37); +lean_dec(x_36); if (lean_is_scalar(x_33)) { x_40 = lean_alloc_ctor(0, 5, 0); } else { @@ -10933,7 +10933,7 @@ if (lean_is_scalar(x_23)) { lean_ctor_set(x_41, 0, x_35); lean_ctor_set(x_41, 1, x_25); lean_ctor_set(x_41, 2, x_26); -lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 3, x_37); lean_ctor_set(x_41, 4, x_40); return x_41; } @@ -10959,8 +10959,8 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_47; x_47 = lean_ctor_get(x_28, 0); lean_inc(x_47); -x_36 = x_45; -x_37 = x_46; +x_36 = x_46; +x_37 = x_45; x_38 = x_47; goto block_42; } @@ -10968,8 +10968,8 @@ else { lean_object* x_48; x_48 = lean_unsigned_to_nat(0u); -x_36 = x_45; -x_37 = x_46; +x_36 = x_46; +x_37 = x_45; x_38 = x_48; goto block_42; } @@ -12097,9 +12097,9 @@ goto block_64; block_57: { lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_nat_add(x_51, x_53); +x_54 = lean_nat_add(x_52, x_53); lean_dec(x_53); -lean_dec(x_51); +lean_dec(x_52); if (lean_is_scalar(x_48)) { x_55 = lean_alloc_ctor(0, 5, 0); } else { @@ -12118,7 +12118,7 @@ if (lean_is_scalar(x_38)) { lean_ctor_set(x_56, 0, x_50); lean_ctor_set(x_56, 1, x_40); lean_ctor_set(x_56, 2, x_41); -lean_ctor_set(x_56, 3, x_52); +lean_ctor_set(x_56, 3, x_51); lean_ctor_set(x_56, 4, x_55); return x_56; } @@ -12144,8 +12144,8 @@ if (lean_obj_tag(x_43) == 0) lean_object* x_62; x_62 = lean_ctor_get(x_43, 0); lean_inc(x_62); -x_51 = x_61; -x_52 = x_60; +x_51 = x_60; +x_52 = x_61; x_53 = x_62; goto block_57; } @@ -12153,8 +12153,8 @@ else { lean_object* x_63; x_63 = lean_unsigned_to_nat(0u); -x_51 = x_61; -x_52 = x_60; +x_51 = x_60; +x_52 = x_61; x_53 = x_63; goto block_57; } @@ -12667,9 +12667,9 @@ goto block_185; block_177: { lean_object* x_174; lean_object* x_175; lean_object* x_176; -x_174 = lean_nat_add(x_171, x_173); +x_174 = lean_nat_add(x_172, x_173); lean_dec(x_173); -lean_dec(x_171); +lean_dec(x_172); if (lean_is_scalar(x_168)) { x_175 = lean_alloc_ctor(0, 5, 0); } else { @@ -12688,7 +12688,7 @@ if (lean_is_scalar(x_158)) { lean_ctor_set(x_176, 0, x_170); lean_ctor_set(x_176, 1, x_161); lean_ctor_set(x_176, 2, x_162); -lean_ctor_set(x_176, 3, x_172); +lean_ctor_set(x_176, 3, x_171); lean_ctor_set(x_176, 4, x_175); return x_176; } @@ -12714,8 +12714,8 @@ if (lean_obj_tag(x_164) == 0) lean_object* x_183; x_183 = lean_ctor_get(x_164, 0); lean_inc(x_183); -x_171 = x_182; -x_172 = x_181; +x_171 = x_181; +x_172 = x_182; x_173 = x_183; goto block_177; } @@ -12723,8 +12723,8 @@ else { lean_object* x_184; x_184 = lean_unsigned_to_nat(0u); -x_171 = x_182; -x_172 = x_181; +x_171 = x_181; +x_172 = x_182; x_173 = x_184; goto block_177; } @@ -13998,9 +13998,9 @@ goto block_196; block_188: { lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_nat_add(x_183, x_184); +x_185 = lean_nat_add(x_182, x_184); lean_dec(x_184); -lean_dec(x_183); +lean_dec(x_182); if (lean_is_scalar(x_178)) { x_186 = lean_alloc_ctor(0, 5, 0); } else { @@ -14019,7 +14019,7 @@ if (lean_is_scalar(x_168)) { lean_ctor_set(x_187, 0, x_181); lean_ctor_set(x_187, 1, x_171); lean_ctor_set(x_187, 2, x_172); -lean_ctor_set(x_187, 3, x_182); +lean_ctor_set(x_187, 3, x_183); lean_ctor_set(x_187, 4, x_186); return x_187; } @@ -14045,8 +14045,8 @@ if (lean_obj_tag(x_174) == 0) lean_object* x_194; x_194 = lean_ctor_get(x_174, 0); lean_inc(x_194); -x_182 = x_192; -x_183 = x_193; +x_182 = x_193; +x_183 = x_192; x_184 = x_194; goto block_188; } @@ -14054,8 +14054,8 @@ else { lean_object* x_195; x_195 = lean_unsigned_to_nat(0u); -x_182 = x_192; -x_183 = x_193; +x_182 = x_193; +x_183 = x_192; x_184 = x_195; goto block_188; } @@ -14732,9 +14732,9 @@ goto block_58; block_51: { lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_nat_add(x_45, x_47); +x_48 = lean_nat_add(x_46, x_47); lean_dec(x_47); -lean_dec(x_45); +lean_dec(x_46); if (lean_is_scalar(x_41)) { x_49 = lean_alloc_ctor(0, 5, 0); } else { @@ -14753,7 +14753,7 @@ if (lean_is_scalar(x_31)) { lean_ctor_set(x_50, 0, x_44); lean_ctor_set(x_50, 1, x_33); lean_ctor_set(x_50, 2, x_34); -lean_ctor_set(x_50, 3, x_46); +lean_ctor_set(x_50, 3, x_45); lean_ctor_set(x_50, 4, x_49); return x_50; } @@ -14779,8 +14779,8 @@ if (lean_obj_tag(x_36) == 0) lean_object* x_56; x_56 = lean_ctor_get(x_36, 0); lean_inc(x_56); -x_45 = x_55; -x_46 = x_54; +x_45 = x_54; +x_46 = x_55; x_47 = x_56; goto block_51; } @@ -14788,8 +14788,8 @@ else { lean_object* x_57; x_57 = lean_unsigned_to_nat(0u); -x_45 = x_55; -x_46 = x_54; +x_45 = x_54; +x_46 = x_55; x_47 = x_57; goto block_51; } @@ -15280,9 +15280,9 @@ goto block_181; block_173: { lean_object* x_164; lean_object* x_165; uint8_t x_166; -x_164 = lean_nat_add(x_162, x_163); +x_164 = lean_nat_add(x_161, x_163); lean_dec(x_163); -lean_dec(x_162); +lean_dec(x_161); lean_inc_ref(x_132); if (lean_is_scalar(x_157)) { x_165 = lean_alloc_ctor(0, 5, 0); @@ -15309,7 +15309,7 @@ lean_dec(x_170); x_171 = lean_ctor_get(x_132, 0); lean_dec(x_171); lean_ctor_set(x_132, 4, x_165); -lean_ctor_set(x_132, 3, x_161); +lean_ctor_set(x_132, 3, x_162); lean_ctor_set(x_132, 2, x_151); lean_ctor_set(x_132, 1, x_150); lean_ctor_set(x_132, 0, x_160); @@ -15323,7 +15323,7 @@ x_172 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_172, 0, x_160); lean_ctor_set(x_172, 1, x_150); lean_ctor_set(x_172, 2, x_151); -lean_ctor_set(x_172, 3, x_161); +lean_ctor_set(x_172, 3, x_162); lean_ctor_set(x_172, 4, x_165); return x_172; } @@ -15350,8 +15350,8 @@ if (lean_obj_tag(x_153) == 0) lean_object* x_179; x_179 = lean_ctor_get(x_153, 0); lean_inc(x_179); -x_161 = x_177; -x_162 = x_178; +x_161 = x_178; +x_162 = x_177; x_163 = x_179; goto block_173; } @@ -15359,8 +15359,8 @@ else { lean_object* x_180; x_180 = lean_unsigned_to_nat(0u); -x_161 = x_177; -x_162 = x_178; +x_161 = x_178; +x_162 = x_177; x_163 = x_180; goto block_173; } @@ -15448,9 +15448,9 @@ goto block_218; block_210: { lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; -x_206 = lean_nat_add(x_204, x_205); +x_206 = lean_nat_add(x_203, x_205); lean_dec(x_205); -lean_dec(x_204); +lean_dec(x_203); lean_inc_ref(x_132); if (lean_is_scalar(x_199)) { x_207 = lean_alloc_ctor(0, 5, 0); @@ -15481,7 +15481,7 @@ if (lean_is_scalar(x_208)) { lean_ctor_set(x_209, 0, x_202); lean_ctor_set(x_209, 1, x_192); lean_ctor_set(x_209, 2, x_193); -lean_ctor_set(x_209, 3, x_203); +lean_ctor_set(x_209, 3, x_204); lean_ctor_set(x_209, 4, x_207); return x_209; } @@ -15507,8 +15507,8 @@ if (lean_obj_tag(x_195) == 0) lean_object* x_216; x_216 = lean_ctor_get(x_195, 0); lean_inc(x_216); -x_203 = x_214; -x_204 = x_215; +x_203 = x_215; +x_204 = x_214; x_205 = x_216; goto block_210; } @@ -15516,8 +15516,8 @@ else { lean_object* x_217; x_217 = lean_unsigned_to_nat(0u); -x_203 = x_214; -x_204 = x_215; +x_203 = x_215; +x_204 = x_214; x_205 = x_217; goto block_210; } @@ -15992,9 +15992,9 @@ goto block_333; block_326: { lean_object* x_323; lean_object* x_324; lean_object* x_325; -x_323 = lean_nat_add(x_321, x_322); +x_323 = lean_nat_add(x_320, x_322); lean_dec(x_322); -lean_dec(x_321); +lean_dec(x_320); if (lean_is_scalar(x_316)) { x_324 = lean_alloc_ctor(0, 5, 0); } else { @@ -16013,7 +16013,7 @@ if (lean_is_scalar(x_306)) { lean_ctor_set(x_325, 0, x_319); lean_ctor_set(x_325, 1, x_308); lean_ctor_set(x_325, 2, x_309); -lean_ctor_set(x_325, 3, x_320); +lean_ctor_set(x_325, 3, x_321); lean_ctor_set(x_325, 4, x_324); return x_325; } @@ -16039,8 +16039,8 @@ if (lean_obj_tag(x_311) == 0) lean_object* x_331; x_331 = lean_ctor_get(x_311, 0); lean_inc(x_331); -x_320 = x_329; -x_321 = x_330; +x_320 = x_330; +x_321 = x_329; x_322 = x_331; goto block_326; } @@ -16048,8 +16048,8 @@ else { lean_object* x_332; x_332 = lean_unsigned_to_nat(0u); -x_320 = x_329; -x_321 = x_330; +x_320 = x_330; +x_321 = x_329; x_322 = x_332; goto block_326; } @@ -20456,9 +20456,9 @@ goto block_156; block_149: { lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_146 = lean_nat_add(x_143, x_145); +x_146 = lean_nat_add(x_144, x_145); lean_dec(x_145); -lean_dec(x_143); +lean_dec(x_144); if (lean_is_scalar(x_140)) { x_147 = lean_alloc_ctor(0, 5, 0); } else { @@ -20477,7 +20477,7 @@ if (lean_is_scalar(x_130)) { lean_ctor_set(x_148, 0, x_142); lean_ctor_set(x_148, 1, x_132); lean_ctor_set(x_148, 2, x_133); -lean_ctor_set(x_148, 3, x_144); +lean_ctor_set(x_148, 3, x_143); lean_ctor_set(x_148, 4, x_147); return x_148; } @@ -20503,8 +20503,8 @@ if (lean_obj_tag(x_135) == 0) lean_object* x_154; x_154 = lean_ctor_get(x_135, 0); lean_inc(x_154); -x_143 = x_153; -x_144 = x_152; +x_143 = x_152; +x_144 = x_153; x_145 = x_154; goto block_149; } @@ -20512,8 +20512,8 @@ else { lean_object* x_155; x_155 = lean_unsigned_to_nat(0u); -x_143 = x_153; -x_144 = x_152; +x_143 = x_152; +x_144 = x_153; x_145 = x_155; goto block_149; } @@ -21613,9 +21613,9 @@ goto block_196; block_189: { lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_186 = lean_nat_add(x_183, x_185); +x_186 = lean_nat_add(x_184, x_185); lean_dec(x_185); -lean_dec(x_183); +lean_dec(x_184); if (lean_is_scalar(x_179)) { x_187 = lean_alloc_ctor(0, 5, 0); } else { @@ -21634,7 +21634,7 @@ if (lean_is_scalar(x_169)) { lean_ctor_set(x_188, 0, x_182); lean_ctor_set(x_188, 1, x_171); lean_ctor_set(x_188, 2, x_172); -lean_ctor_set(x_188, 3, x_184); +lean_ctor_set(x_188, 3, x_183); lean_ctor_set(x_188, 4, x_187); return x_188; } @@ -21660,8 +21660,8 @@ if (lean_obj_tag(x_174) == 0) lean_object* x_194; x_194 = lean_ctor_get(x_174, 0); lean_inc(x_194); -x_183 = x_193; -x_184 = x_192; +x_183 = x_192; +x_184 = x_193; x_185 = x_194; goto block_189; } @@ -21669,8 +21669,8 @@ else { lean_object* x_195; x_195 = lean_unsigned_to_nat(0u); -x_183 = x_193; -x_184 = x_192; +x_183 = x_192; +x_184 = x_193; x_185 = x_195; goto block_189; } @@ -22893,9 +22893,9 @@ goto block_51; block_44: { lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_nat_add(x_39, x_40); +x_41 = lean_nat_add(x_38, x_40); lean_dec(x_40); -lean_dec(x_39); +lean_dec(x_38); if (lean_is_scalar(x_35)) { x_42 = lean_alloc_ctor(0, 5, 0); } else { @@ -22914,7 +22914,7 @@ if (lean_is_scalar(x_25)) { lean_ctor_set(x_43, 0, x_37); lean_ctor_set(x_43, 1, x_27); lean_ctor_set(x_43, 2, x_28); -lean_ctor_set(x_43, 3, x_38); +lean_ctor_set(x_43, 3, x_39); lean_ctor_set(x_43, 4, x_42); return x_43; } @@ -22940,8 +22940,8 @@ if (lean_obj_tag(x_30) == 0) lean_object* x_49; x_49 = lean_ctor_get(x_30, 0); lean_inc(x_49); -x_38 = x_47; -x_39 = x_48; +x_38 = x_48; +x_39 = x_47; x_40 = x_49; goto block_44; } @@ -22949,8 +22949,8 @@ else { lean_object* x_50; x_50 = lean_unsigned_to_nat(0u); -x_38 = x_47; -x_39 = x_48; +x_38 = x_48; +x_39 = x_47; x_40 = x_50; goto block_44; } @@ -23526,9 +23526,9 @@ goto block_190; block_183: { lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_180 = lean_nat_add(x_178, x_179); +x_180 = lean_nat_add(x_177, x_179); lean_dec(x_179); -lean_dec(x_178); +lean_dec(x_177); if (lean_is_scalar(x_174)) { x_181 = lean_alloc_ctor(0, 5, 0); } else { @@ -23547,7 +23547,7 @@ if (lean_is_scalar(x_164)) { lean_ctor_set(x_182, 0, x_176); lean_ctor_set(x_182, 1, x_166); lean_ctor_set(x_182, 2, x_167); -lean_ctor_set(x_182, 3, x_177); +lean_ctor_set(x_182, 3, x_178); lean_ctor_set(x_182, 4, x_181); return x_182; } @@ -23573,8 +23573,8 @@ if (lean_obj_tag(x_169) == 0) lean_object* x_188; x_188 = lean_ctor_get(x_169, 0); lean_inc(x_188); -x_177 = x_186; -x_178 = x_187; +x_177 = x_187; +x_178 = x_186; x_179 = x_188; goto block_183; } @@ -23582,8 +23582,8 @@ else { lean_object* x_189; x_189 = lean_unsigned_to_nat(0u); -x_177 = x_186; -x_178 = x_187; +x_177 = x_187; +x_178 = x_186; x_179 = x_189; goto block_183; } @@ -25400,9 +25400,9 @@ goto block_52; block_45: { lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_nat_add(x_40, x_41); +x_42 = lean_nat_add(x_39, x_41); lean_dec(x_41); -lean_dec(x_40); +lean_dec(x_39); if (lean_is_scalar(x_35)) { x_43 = lean_alloc_ctor(0, 5, 0); } else { @@ -25421,7 +25421,7 @@ if (lean_is_scalar(x_25)) { lean_ctor_set(x_44, 0, x_38); lean_ctor_set(x_44, 1, x_27); lean_ctor_set(x_44, 2, x_28); -lean_ctor_set(x_44, 3, x_39); +lean_ctor_set(x_44, 3, x_40); lean_ctor_set(x_44, 4, x_43); return x_44; } @@ -25447,8 +25447,8 @@ if (lean_obj_tag(x_30) == 0) lean_object* x_50; x_50 = lean_ctor_get(x_30, 0); lean_inc(x_50); -x_39 = x_48; -x_40 = x_49; +x_39 = x_49; +x_40 = x_48; x_41 = x_50; goto block_45; } @@ -25456,8 +25456,8 @@ else { lean_object* x_51; x_51 = lean_unsigned_to_nat(0u); -x_39 = x_48; -x_40 = x_49; +x_39 = x_49; +x_40 = x_48; x_41 = x_51; goto block_45; } @@ -26048,9 +26048,9 @@ goto block_199; block_192: { lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_nat_add(x_187, x_188); +x_189 = lean_nat_add(x_186, x_188); lean_dec(x_188); -lean_dec(x_187); +lean_dec(x_186); if (lean_is_scalar(x_182)) { x_190 = lean_alloc_ctor(0, 5, 0); } else { @@ -26069,7 +26069,7 @@ if (lean_is_scalar(x_172)) { lean_ctor_set(x_191, 0, x_185); lean_ctor_set(x_191, 1, x_174); lean_ctor_set(x_191, 2, x_175); -lean_ctor_set(x_191, 3, x_186); +lean_ctor_set(x_191, 3, x_187); lean_ctor_set(x_191, 4, x_190); return x_191; } @@ -26095,8 +26095,8 @@ if (lean_obj_tag(x_177) == 0) lean_object* x_197; x_197 = lean_ctor_get(x_177, 0); lean_inc(x_197); -x_186 = x_195; -x_187 = x_196; +x_186 = x_196; +x_187 = x_195; x_188 = x_197; goto block_192; } @@ -26104,8 +26104,8 @@ else { lean_object* x_198; x_198 = lean_unsigned_to_nat(0u); -x_186 = x_195; -x_187 = x_196; +x_186 = x_196; +x_187 = x_195; x_188 = x_198; goto block_192; } @@ -33386,9 +33386,9 @@ goto block_204; block_196: { lean_object* x_187; lean_object* x_188; uint8_t x_189; -x_187 = lean_nat_add(x_184, x_186); +x_187 = lean_nat_add(x_185, x_186); lean_dec(x_186); -lean_dec(x_184); +lean_dec(x_185); lean_inc_ref(x_154); if (lean_is_scalar(x_180)) { x_188 = lean_alloc_ctor(0, 5, 0); @@ -33415,7 +33415,7 @@ lean_dec(x_193); x_194 = lean_ctor_get(x_154, 0); lean_dec(x_194); lean_ctor_set(x_154, 4, x_188); -lean_ctor_set(x_154, 3, x_185); +lean_ctor_set(x_154, 3, x_184); lean_ctor_set(x_154, 2, x_174); lean_ctor_set(x_154, 1, x_173); lean_ctor_set(x_154, 0, x_183); @@ -33429,7 +33429,7 @@ x_195 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_195, 0, x_183); lean_ctor_set(x_195, 1, x_173); lean_ctor_set(x_195, 2, x_174); -lean_ctor_set(x_195, 3, x_185); +lean_ctor_set(x_195, 3, x_184); lean_ctor_set(x_195, 4, x_188); return x_195; } @@ -33456,8 +33456,8 @@ if (lean_obj_tag(x_176) == 0) lean_object* x_202; x_202 = lean_ctor_get(x_176, 0); lean_inc(x_202); -x_184 = x_201; -x_185 = x_200; +x_184 = x_200; +x_185 = x_201; x_186 = x_202; goto block_196; } @@ -33465,8 +33465,8 @@ else { lean_object* x_203; x_203 = lean_unsigned_to_nat(0u); -x_184 = x_201; -x_185 = x_200; +x_184 = x_200; +x_185 = x_201; x_186 = x_203; goto block_196; } @@ -33594,9 +33594,9 @@ goto block_247; block_239: { lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; -x_235 = lean_nat_add(x_232, x_234); +x_235 = lean_nat_add(x_233, x_234); lean_dec(x_234); -lean_dec(x_232); +lean_dec(x_233); lean_inc_ref(x_154); if (lean_is_scalar(x_228)) { x_236 = lean_alloc_ctor(0, 5, 0); @@ -33627,7 +33627,7 @@ if (lean_is_scalar(x_237)) { lean_ctor_set(x_238, 0, x_231); lean_ctor_set(x_238, 1, x_221); lean_ctor_set(x_238, 2, x_222); -lean_ctor_set(x_238, 3, x_233); +lean_ctor_set(x_238, 3, x_232); lean_ctor_set(x_238, 4, x_236); return x_238; } @@ -33653,8 +33653,8 @@ if (lean_obj_tag(x_224) == 0) lean_object* x_245; x_245 = lean_ctor_get(x_224, 0); lean_inc(x_245); -x_232 = x_244; -x_233 = x_243; +x_232 = x_243; +x_233 = x_244; x_234 = x_245; goto block_239; } @@ -33662,8 +33662,8 @@ else { lean_object* x_246; x_246 = lean_unsigned_to_nat(0u); -x_232 = x_244; -x_233 = x_243; +x_232 = x_243; +x_233 = x_244; x_234 = x_246; goto block_239; } @@ -34715,9 +34715,9 @@ goto block_484; block_476: { lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; -x_472 = lean_nat_add(x_469, x_471); +x_472 = lean_nat_add(x_470, x_471); lean_dec(x_471); -lean_dec(x_469); +lean_dec(x_470); lean_inc_ref(x_444); if (lean_is_scalar(x_465)) { x_473 = lean_alloc_ctor(0, 5, 0); @@ -34748,7 +34748,7 @@ if (lean_is_scalar(x_474)) { lean_ctor_set(x_475, 0, x_468); lean_ctor_set(x_475, 1, x_458); lean_ctor_set(x_475, 2, x_459); -lean_ctor_set(x_475, 3, x_470); +lean_ctor_set(x_475, 3, x_469); lean_ctor_set(x_475, 4, x_473); return x_475; } @@ -34774,8 +34774,8 @@ if (lean_obj_tag(x_461) == 0) lean_object* x_482; x_482 = lean_ctor_get(x_461, 0); lean_inc(x_482); -x_469 = x_481; -x_470 = x_480; +x_469 = x_480; +x_470 = x_481; x_471 = x_482; goto block_476; } @@ -34783,8 +34783,8 @@ else { lean_object* x_483; x_483 = lean_unsigned_to_nat(0u); -x_469 = x_481; -x_470 = x_480; +x_469 = x_480; +x_470 = x_481; x_471 = x_483; goto block_476; } @@ -36346,9 +36346,9 @@ goto block_186; block_178: { lean_object* x_169; lean_object* x_170; uint8_t x_171; -x_169 = lean_nat_add(x_166, x_168); +x_169 = lean_nat_add(x_167, x_168); lean_dec(x_168); -lean_dec(x_166); +lean_dec(x_167); lean_inc_ref(x_138); if (lean_is_scalar(x_163)) { x_170 = lean_alloc_ctor(0, 5, 0); @@ -36375,7 +36375,7 @@ lean_dec(x_175); x_176 = lean_ctor_get(x_138, 0); lean_dec(x_176); lean_ctor_set(x_138, 4, x_170); -lean_ctor_set(x_138, 3, x_167); +lean_ctor_set(x_138, 3, x_166); lean_ctor_set(x_138, 2, x_157); lean_ctor_set(x_138, 1, x_156); lean_ctor_set(x_138, 0, x_165); @@ -36389,7 +36389,7 @@ x_177 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_177, 0, x_165); lean_ctor_set(x_177, 1, x_156); lean_ctor_set(x_177, 2, x_157); -lean_ctor_set(x_177, 3, x_167); +lean_ctor_set(x_177, 3, x_166); lean_ctor_set(x_177, 4, x_170); return x_177; } @@ -36416,8 +36416,8 @@ if (lean_obj_tag(x_159) == 0) lean_object* x_184; x_184 = lean_ctor_get(x_159, 0); lean_inc(x_184); -x_166 = x_183; -x_167 = x_182; +x_166 = x_182; +x_167 = x_183; x_168 = x_184; goto block_178; } @@ -36425,8 +36425,8 @@ else { lean_object* x_185; x_185 = lean_unsigned_to_nat(0u); -x_166 = x_183; -x_167 = x_182; +x_166 = x_182; +x_167 = x_183; x_168 = x_185; goto block_178; } @@ -36512,9 +36512,9 @@ goto block_221; block_213: { lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_209 = lean_nat_add(x_206, x_208); +x_209 = lean_nat_add(x_207, x_208); lean_dec(x_208); -lean_dec(x_206); +lean_dec(x_207); lean_inc_ref(x_138); if (lean_is_scalar(x_203)) { x_210 = lean_alloc_ctor(0, 5, 0); @@ -36545,7 +36545,7 @@ if (lean_is_scalar(x_211)) { lean_ctor_set(x_212, 0, x_205); lean_ctor_set(x_212, 1, x_196); lean_ctor_set(x_212, 2, x_197); -lean_ctor_set(x_212, 3, x_207); +lean_ctor_set(x_212, 3, x_206); lean_ctor_set(x_212, 4, x_210); return x_212; } @@ -36571,8 +36571,8 @@ if (lean_obj_tag(x_199) == 0) lean_object* x_219; x_219 = lean_ctor_get(x_199, 0); lean_inc(x_219); -x_206 = x_218; -x_207 = x_217; +x_206 = x_217; +x_207 = x_218; x_208 = x_219; goto block_213; } @@ -36580,8 +36580,8 @@ else { lean_object* x_220; x_220 = lean_unsigned_to_nat(0u); -x_206 = x_218; -x_207 = x_217; +x_206 = x_217; +x_207 = x_218; x_208 = x_220; goto block_213; } @@ -37536,9 +37536,9 @@ goto block_431; block_423: { lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; -x_419 = lean_nat_add(x_416, x_418); +x_419 = lean_nat_add(x_417, x_418); lean_dec(x_418); -lean_dec(x_416); +lean_dec(x_417); lean_inc_ref(x_393); if (lean_is_scalar(x_413)) { x_420 = lean_alloc_ctor(0, 5, 0); @@ -37569,7 +37569,7 @@ if (lean_is_scalar(x_421)) { lean_ctor_set(x_422, 0, x_415); lean_ctor_set(x_422, 1, x_406); lean_ctor_set(x_422, 2, x_407); -lean_ctor_set(x_422, 3, x_417); +lean_ctor_set(x_422, 3, x_416); lean_ctor_set(x_422, 4, x_420); return x_422; } @@ -37595,8 +37595,8 @@ if (lean_obj_tag(x_409) == 0) lean_object* x_429; x_429 = lean_ctor_get(x_409, 0); lean_inc(x_429); -x_416 = x_428; -x_417 = x_427; +x_416 = x_427; +x_417 = x_428; x_418 = x_429; goto block_423; } @@ -37604,8 +37604,8 @@ else { lean_object* x_430; x_430 = lean_unsigned_to_nat(0u); -x_416 = x_428; -x_417 = x_427; +x_416 = x_427; +x_417 = x_428; x_418 = x_430; goto block_423; } @@ -38089,9 +38089,9 @@ goto block_68; block_61: { lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_nat_add(x_55, x_57); +x_58 = lean_nat_add(x_56, x_57); lean_dec(x_57); -lean_dec(x_55); +lean_dec(x_56); if (lean_is_scalar(x_51)) { x_59 = lean_alloc_ctor(0, 5, 0); } else { @@ -38110,7 +38110,7 @@ if (lean_is_scalar(x_41)) { lean_ctor_set(x_60, 0, x_54); lean_ctor_set(x_60, 1, x_43); lean_ctor_set(x_60, 2, x_44); -lean_ctor_set(x_60, 3, x_56); +lean_ctor_set(x_60, 3, x_55); lean_ctor_set(x_60, 4, x_59); return x_60; } @@ -38136,8 +38136,8 @@ if (lean_obj_tag(x_46) == 0) lean_object* x_66; x_66 = lean_ctor_get(x_46, 0); lean_inc(x_66); -x_55 = x_65; -x_56 = x_64; +x_55 = x_64; +x_56 = x_65; x_57 = x_66; goto block_61; } @@ -38145,8 +38145,8 @@ else { lean_object* x_67; x_67 = lean_unsigned_to_nat(0u); -x_55 = x_65; -x_56 = x_64; +x_55 = x_64; +x_56 = x_65; x_57 = x_67; goto block_61; } @@ -38668,9 +38668,9 @@ goto block_204; block_196: { lean_object* x_187; lean_object* x_188; uint8_t x_189; -x_187 = lean_nat_add(x_185, x_186); +x_187 = lean_nat_add(x_184, x_186); lean_dec(x_186); -lean_dec(x_185); +lean_dec(x_184); lean_inc_ref(x_154); if (lean_is_scalar(x_180)) { x_188 = lean_alloc_ctor(0, 5, 0); @@ -38697,7 +38697,7 @@ lean_dec(x_193); x_194 = lean_ctor_get(x_154, 0); lean_dec(x_194); lean_ctor_set(x_154, 4, x_188); -lean_ctor_set(x_154, 3, x_184); +lean_ctor_set(x_154, 3, x_185); lean_ctor_set(x_154, 2, x_174); lean_ctor_set(x_154, 1, x_173); lean_ctor_set(x_154, 0, x_183); @@ -38711,7 +38711,7 @@ x_195 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_195, 0, x_183); lean_ctor_set(x_195, 1, x_173); lean_ctor_set(x_195, 2, x_174); -lean_ctor_set(x_195, 3, x_184); +lean_ctor_set(x_195, 3, x_185); lean_ctor_set(x_195, 4, x_188); return x_195; } @@ -38738,8 +38738,8 @@ if (lean_obj_tag(x_176) == 0) lean_object* x_202; x_202 = lean_ctor_get(x_176, 0); lean_inc(x_202); -x_184 = x_200; -x_185 = x_201; +x_184 = x_201; +x_185 = x_200; x_186 = x_202; goto block_196; } @@ -38747,8 +38747,8 @@ else { lean_object* x_203; x_203 = lean_unsigned_to_nat(0u); -x_184 = x_200; -x_185 = x_201; +x_184 = x_201; +x_185 = x_200; x_186 = x_203; goto block_196; } @@ -38876,9 +38876,9 @@ goto block_247; block_239: { lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; -x_235 = lean_nat_add(x_233, x_234); +x_235 = lean_nat_add(x_232, x_234); lean_dec(x_234); -lean_dec(x_233); +lean_dec(x_232); lean_inc_ref(x_154); if (lean_is_scalar(x_228)) { x_236 = lean_alloc_ctor(0, 5, 0); @@ -38909,7 +38909,7 @@ if (lean_is_scalar(x_237)) { lean_ctor_set(x_238, 0, x_231); lean_ctor_set(x_238, 1, x_221); lean_ctor_set(x_238, 2, x_222); -lean_ctor_set(x_238, 3, x_232); +lean_ctor_set(x_238, 3, x_233); lean_ctor_set(x_238, 4, x_236); return x_238; } @@ -38935,8 +38935,8 @@ if (lean_obj_tag(x_224) == 0) lean_object* x_245; x_245 = lean_ctor_get(x_224, 0); lean_inc(x_245); -x_232 = x_243; -x_233 = x_244; +x_232 = x_244; +x_233 = x_243; x_234 = x_245; goto block_239; } @@ -38944,8 +38944,8 @@ else { lean_object* x_246; x_246 = lean_unsigned_to_nat(0u); -x_232 = x_243; -x_233 = x_244; +x_232 = x_244; +x_233 = x_243; x_234 = x_246; goto block_239; } @@ -39551,9 +39551,9 @@ goto block_397; block_390: { lean_object* x_387; lean_object* x_388; lean_object* x_389; -x_387 = lean_nat_add(x_384, x_386); +x_387 = lean_nat_add(x_385, x_386); lean_dec(x_386); -lean_dec(x_384); +lean_dec(x_385); if (lean_is_scalar(x_380)) { x_388 = lean_alloc_ctor(0, 5, 0); } else { @@ -39572,7 +39572,7 @@ if (lean_is_scalar(x_370)) { lean_ctor_set(x_389, 0, x_383); lean_ctor_set(x_389, 1, x_372); lean_ctor_set(x_389, 2, x_373); -lean_ctor_set(x_389, 3, x_385); +lean_ctor_set(x_389, 3, x_384); lean_ctor_set(x_389, 4, x_388); return x_389; } @@ -39598,8 +39598,8 @@ if (lean_obj_tag(x_375) == 0) lean_object* x_395; x_395 = lean_ctor_get(x_375, 0); lean_inc(x_395); -x_384 = x_394; -x_385 = x_393; +x_384 = x_393; +x_385 = x_394; x_386 = x_395; goto block_390; } @@ -39607,8 +39607,8 @@ else { lean_object* x_396; x_396 = lean_unsigned_to_nat(0u); -x_384 = x_394; -x_385 = x_393; +x_384 = x_393; +x_385 = x_394; x_386 = x_396; goto block_390; } @@ -39997,9 +39997,9 @@ goto block_484; block_476: { lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; -x_472 = lean_nat_add(x_470, x_471); +x_472 = lean_nat_add(x_469, x_471); lean_dec(x_471); -lean_dec(x_470); +lean_dec(x_469); lean_inc_ref(x_444); if (lean_is_scalar(x_465)) { x_473 = lean_alloc_ctor(0, 5, 0); @@ -40030,7 +40030,7 @@ if (lean_is_scalar(x_474)) { lean_ctor_set(x_475, 0, x_468); lean_ctor_set(x_475, 1, x_458); lean_ctor_set(x_475, 2, x_459); -lean_ctor_set(x_475, 3, x_469); +lean_ctor_set(x_475, 3, x_470); lean_ctor_set(x_475, 4, x_473); return x_475; } @@ -40056,8 +40056,8 @@ if (lean_obj_tag(x_461) == 0) lean_object* x_482; x_482 = lean_ctor_get(x_461, 0); lean_inc(x_482); -x_469 = x_480; -x_470 = x_481; +x_469 = x_481; +x_470 = x_480; x_471 = x_482; goto block_476; } @@ -40065,8 +40065,8 @@ else { lean_object* x_483; x_483 = lean_unsigned_to_nat(0u); -x_469 = x_480; -x_470 = x_481; +x_469 = x_481; +x_470 = x_480; x_471 = x_483; goto block_476; } 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 3624f5a74f2e..cdc6ae4c2479 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 @@ -3778,9 +3778,9 @@ goto block_44; { lean_object* x_6; lean_object* x_7; x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 0, x_4); lean_ctor_set(x_6, 1, x_5); -x_7 = l_Std_Sat_AIG_mkGateCached___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__5(x_4, x_6); +x_7 = l_Std_Sat_AIG_mkGateCached___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__5(x_3, x_6); return x_7; } block_23: @@ -3796,8 +3796,8 @@ if (x_13 == 0) uint8_t x_14; x_14 = 1; lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_14); -x_3 = x_11; -x_4 = x_10; +x_3 = x_10; +x_4 = x_11; x_5 = x_9; goto block_8; } @@ -3811,8 +3811,8 @@ x_16 = 1; x_17 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_17, 0, x_15); lean_ctor_set_uint8(x_17, sizeof(void*)*1, x_16); -x_3 = x_11; -x_4 = x_10; +x_3 = x_10; +x_4 = x_11; x_5 = x_17; goto block_8; } @@ -3826,8 +3826,8 @@ if (x_18 == 0) uint8_t x_19; x_19 = 0; lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_19); -x_3 = x_11; -x_4 = x_10; +x_3 = x_10; +x_4 = x_11; x_5 = x_9; goto block_8; } @@ -3841,8 +3841,8 @@ x_21 = 0; x_22 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_22, 0, x_20); lean_ctor_set_uint8(x_22, sizeof(void*)*1, x_21); -x_3 = x_11; -x_4 = x_10; +x_3 = x_10; +x_4 = x_11; x_5 = x_22; goto block_8; } @@ -4319,7 +4319,7 @@ return x_6; LEAN_EXPORT lean_object* l_Std_Sat_AIG_mkBEqCached___at___00Std_Tactic_BVDecide_BVPred_mkEq___at___00Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__13_spec__27_spec__38(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; uint8_t x_48; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; uint8_t x_48; x_48 = !lean_is_exclusive(x_2); if (x_48 == 0) { @@ -4388,9 +4388,9 @@ if (lean_is_scalar(x_56)) { lean_ctor_set(x_62, 0, x_52); lean_ctor_set_uint8(x_62, sizeof(void*)*1, x_61); x_24 = x_54; -x_25 = x_60; -x_26 = x_59; -x_27 = x_55; +x_25 = x_59; +x_26 = x_55; +x_27 = x_60; x_28 = x_62; goto block_47; } @@ -4411,9 +4411,9 @@ if (lean_is_scalar(x_56)) { lean_ctor_set(x_66, 0, x_52); lean_ctor_set_uint8(x_66, sizeof(void*)*1, x_65); x_24 = x_54; -x_25 = x_64; -x_26 = x_63; -x_27 = x_55; +x_25 = x_63; +x_26 = x_55; +x_27 = x_64; x_28 = x_66; goto block_47; } @@ -4488,9 +4488,9 @@ if (lean_is_scalar(x_77)) { lean_ctor_set(x_83, 0, x_73); lean_ctor_set_uint8(x_83, sizeof(void*)*1, x_82); x_24 = x_75; -x_25 = x_81; -x_26 = x_80; -x_27 = x_76; +x_25 = x_80; +x_26 = x_76; +x_27 = x_81; x_28 = x_83; goto block_47; } @@ -4511,9 +4511,9 @@ if (lean_is_scalar(x_77)) { lean_ctor_set(x_87, 0, x_73); lean_ctor_set_uint8(x_87, sizeof(void*)*1, x_86); x_24 = x_75; -x_25 = x_85; -x_26 = x_84; -x_27 = x_76; +x_25 = x_84; +x_26 = x_76; +x_27 = x_85; x_28 = x_87; goto block_47; } @@ -4605,9 +4605,9 @@ if (lean_is_scalar(x_101)) { lean_ctor_set(x_107, 0, x_96); lean_ctor_set_uint8(x_107, sizeof(void*)*1, x_106); x_24 = x_99; -x_25 = x_105; -x_26 = x_104; -x_27 = x_100; +x_25 = x_104; +x_26 = x_100; +x_27 = x_105; x_28 = x_107; goto block_47; } @@ -4628,9 +4628,9 @@ if (lean_is_scalar(x_101)) { lean_ctor_set(x_111, 0, x_96); lean_ctor_set_uint8(x_111, sizeof(void*)*1, x_110); x_24 = x_99; -x_25 = x_109; -x_26 = x_108; -x_27 = x_100; +x_25 = x_108; +x_26 = x_100; +x_27 = x_109; x_28 = x_111; goto block_47; } @@ -4715,12 +4715,12 @@ goto block_8; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; x_29 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_29, 0, x_24); -lean_ctor_set_uint8(x_29, sizeof(void*)*1, x_27); +lean_ctor_set_uint8(x_29, sizeof(void*)*1, x_26); x_30 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_30, 0, x_28); lean_ctor_set(x_30, 1, x_29); -x_31 = l_Std_Sat_AIG_mkGateCached___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__5(x_26, x_30); -x_32 = lean_ctor_get_uint8(x_25, sizeof(void*)*1); +x_31 = l_Std_Sat_AIG_mkGateCached___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__5(x_25, x_30); +x_32 = lean_ctor_get_uint8(x_27, sizeof(void*)*1); if (x_32 == 0) { lean_object* x_33; lean_object* x_34; uint8_t x_35; @@ -4729,23 +4729,23 @@ lean_inc_ref(x_33); x_34 = lean_ctor_get(x_31, 1); lean_inc_ref(x_34); lean_dec_ref(x_31); -x_35 = !lean_is_exclusive(x_25); +x_35 = !lean_is_exclusive(x_27); if (x_35 == 0) { uint8_t x_36; x_36 = 1; -lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_36); +lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_36); x_9 = x_34; x_10 = x_33; -x_11 = x_25; +x_11 = x_27; goto block_23; } else { lean_object* x_37; uint8_t x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_25, 0); +x_37 = lean_ctor_get(x_27, 0); lean_inc(x_37); -lean_dec(x_25); +lean_dec(x_27); x_38 = 1; x_39 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_39, 0, x_37); @@ -4764,23 +4764,23 @@ lean_inc_ref(x_40); x_41 = lean_ctor_get(x_31, 1); lean_inc_ref(x_41); lean_dec_ref(x_31); -x_42 = !lean_is_exclusive(x_25); +x_42 = !lean_is_exclusive(x_27); if (x_42 == 0) { uint8_t x_43; x_43 = 0; -lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_43); +lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_43); x_9 = x_41; x_10 = x_40; -x_11 = x_25; +x_11 = x_27; goto block_23; } else { lean_object* x_44; uint8_t x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_25, 0); +x_44 = lean_ctor_get(x_27, 0); lean_inc(x_44); -lean_dec(x_25); +lean_dec(x_27); x_45 = 0; x_46 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_46, 0, x_44); @@ -7687,9 +7687,9 @@ goto block_54; 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_alloc_ctor(0, 3, 0); lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_7); +lean_ctor_set(x_10, 1, x_8); lean_ctor_set(x_10, 2, x_6); -x_11 = l_Std_Sat_AIG_RefVec_ite___at___00Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__13_spec__29(x_1, x_8, x_10); +x_11 = l_Std_Sat_AIG_RefVec_ite___at___00Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at___00Std_Tactic_BVDecide_BVExpr_bitblast_go_spec__13_spec__29(x_1, x_7, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc_ref(x_12); x_13 = lean_ctor_get(x_11, 1); @@ -7745,8 +7745,8 @@ lean_object* x_35; x_35 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_35, 0, x_31); lean_ctor_set_uint8(x_35, sizeof(void*)*1, x_18); -x_7 = x_28; -x_8 = x_27; +x_7 = x_27; +x_8 = x_28; x_9 = x_35; goto block_17; } @@ -7756,8 +7756,8 @@ lean_object* x_36; x_36 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_36, 0, x_31); lean_ctor_set_uint8(x_36, sizeof(void*)*1, x_21); -x_7 = x_28; -x_8 = x_27; +x_7 = x_27; +x_8 = x_28; x_9 = x_36; goto block_17; } @@ -7793,8 +7793,8 @@ lean_object* x_49; x_49 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_49, 0, x_45); lean_ctor_set_uint8(x_49, sizeof(void*)*1, x_18); -x_7 = x_42; -x_8 = x_41; +x_7 = x_41; +x_8 = x_42; x_9 = x_49; goto block_17; } @@ -7804,8 +7804,8 @@ lean_object* x_50; x_50 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_50, 0, x_45); lean_ctor_set_uint8(x_50, sizeof(void*)*1, x_21); -x_7 = x_42; -x_8 = x_41; +x_7 = x_41; +x_8 = x_42; x_9 = x_50; goto block_17; } diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Mul.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Mul.c index 36dbb397ee63..5ed55cf7e326 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Mul.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Mul.c @@ -91,11 +91,11 @@ goto block_56; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_12 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_9); +lean_ctor_set(x_12, 1, x_10); lean_ctor_set(x_12, 2, x_8); lean_inc_ref(x_2); lean_inc_ref(x_1); -x_13 = l_Std_Sat_AIG_RefVec_ite___redArg(x_1, x_2, x_3, x_10, x_12); +x_13 = l_Std_Sat_AIG_RefVec_ite___redArg(x_1, x_2, x_3, x_9, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc_ref(x_14); x_15 = lean_ctor_get(x_13, 1); @@ -153,8 +153,8 @@ lean_object* x_37; x_37 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_37, 0, x_33); lean_ctor_set_uint8(x_37, sizeof(void*)*1, x_20); -x_9 = x_30; -x_10 = x_29; +x_9 = x_29; +x_10 = x_30; x_11 = x_37; goto block_19; } @@ -164,8 +164,8 @@ lean_object* x_38; x_38 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_38, 0, x_33); lean_ctor_set_uint8(x_38, sizeof(void*)*1, x_23); -x_9 = x_30; -x_10 = x_29; +x_9 = x_29; +x_10 = x_30; x_11 = x_38; goto block_19; } @@ -203,8 +203,8 @@ lean_object* x_51; x_51 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_51, 0, x_47); lean_ctor_set_uint8(x_51, sizeof(void*)*1, x_20); -x_9 = x_44; -x_10 = x_43; +x_9 = x_43; +x_10 = x_44; x_11 = x_51; goto block_19; } @@ -214,8 +214,8 @@ lean_object* x_52; x_52 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_52, 0, x_47); lean_ctor_set_uint8(x_52, sizeof(void*)*1, x_23); -x_9 = x_44; -x_10 = x_43; +x_9 = x_43; +x_10 = x_44; x_11 = x_52; goto block_19; } diff --git a/stage0/stdlib/Std/Time/Format/Basic.c b/stage0/stdlib/Std/Time/Format/Basic.c index fcbcf7b3f970..f0104db89568 100644 --- a/stage0/stdlib/Std/Time/Format/Basic.c +++ b/stage0/stdlib/Std/Time/Format/Basic.c @@ -50077,14 +50077,14 @@ goto block_162; block_13: { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_string_append(x_6, x_7); +x_8 = lean_string_append(x_5, x_7); lean_dec_ref(x_7); x_9 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset___closed__0; x_10 = lean_string_append(x_8, x_9); x_11 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_11, 0, x_10); x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_5); +lean_ctor_set(x_12, 0, x_6); lean_ctor_set(x_12, 1, x_11); return x_12; } @@ -50105,11 +50105,11 @@ return x_21; block_30: { lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_int_add(x_25, x_26); +x_27 = lean_int_add(x_24, x_26); lean_dec(x_26); -lean_dec(x_25); -x_28 = lean_int_mul(x_27, x_24); lean_dec(x_24); +x_28 = lean_int_mul(x_27, x_25); +lean_dec(x_25); lean_dec(x_27); x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_23); @@ -50119,32 +50119,32 @@ return x_29; block_42: { lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_nat_to_int(x_35); +x_37 = lean_nat_to_int(x_33); x_38 = lean_int_mul(x_36, x_37); lean_dec(x_37); lean_dec(x_36); -x_39 = lean_int_add(x_34, x_38); +x_39 = lean_int_add(x_35, x_38); lean_dec(x_38); -lean_dec(x_34); -if (lean_obj_tag(x_33) == 0) +lean_dec(x_35); +if (lean_obj_tag(x_32) == 0) { lean_object* x_40; x_40 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; x_23 = x_31; -x_24 = x_32; -x_25 = x_39; +x_24 = x_39; +x_25 = x_34; x_26 = x_40; goto block_30; } else { lean_object* x_41; -x_41 = lean_ctor_get(x_33, 0); +x_41 = lean_ctor_get(x_32, 0); lean_inc(x_41); -lean_dec_ref(x_33); +lean_dec_ref(x_32); x_23 = x_31; -x_24 = x_32; -x_25 = x_39; +x_24 = x_39; +x_25 = x_34; x_26 = x_41; goto block_30; } @@ -50153,31 +50153,31 @@ goto block_30; { lean_object* x_49; lean_object* x_50; x_49 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__3; -x_50 = lean_int_mul(x_46, x_49); -lean_dec(x_46); -if (lean_obj_tag(x_45) == 0) +x_50 = lean_int_mul(x_47, x_49); +lean_dec(x_47); +if (lean_obj_tag(x_43) == 0) { lean_object* x_51; x_51 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; x_31 = x_48; -x_32 = x_43; +x_32 = x_45; x_33 = x_44; -x_34 = x_50; -x_35 = x_47; +x_34 = x_46; +x_35 = x_50; x_36 = x_51; goto block_42; } else { lean_object* x_52; -x_52 = lean_ctor_get(x_45, 0); +x_52 = lean_ctor_get(x_43, 0); lean_inc(x_52); -lean_dec_ref(x_45); +lean_dec_ref(x_43); x_31 = x_48; -x_32 = x_43; +x_32 = x_45; x_33 = x_44; -x_34 = x_50; -x_35 = x_47; +x_34 = x_46; +x_35 = x_50; x_36 = x_52; goto block_42; } @@ -50188,7 +50188,7 @@ lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; x_60 = lean_unsigned_to_nat(1u); x_61 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset___closed__1; x_62 = lean_box(x_2); -x_63 = lean_apply_3(x_57, x_61, x_62, x_59); +x_63 = lean_apply_3(x_55, x_61, x_62, x_59); if (lean_obj_tag(x_63) == 0) { lean_object* x_64; @@ -50206,9 +50206,9 @@ x_68 = lean_int_dec_lt(x_67, x_66); if (x_68 == 0) { x_43 = x_54; -x_44 = x_64; -x_45 = x_56; -x_46 = x_55; +x_44 = x_56; +x_45 = x_64; +x_46 = x_57; x_47 = x_58; x_48 = x_65; goto block_53; @@ -50219,8 +50219,8 @@ lean_object* x_69; lean_object* x_70; uint8_t x_71; lean_inc(x_66); lean_dec_ref(x_64); lean_dec(x_58); +lean_dec(x_57); lean_dec(x_56); -lean_dec(x_55); lean_dec(x_54); x_69 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset___closed__3; x_70 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; @@ -50263,9 +50263,9 @@ x_80 = lean_ctor_get(x_63, 0); lean_inc(x_80); lean_dec_ref(x_63); x_43 = x_54; -x_44 = x_64; -x_45 = x_56; -x_46 = x_55; +x_44 = x_56; +x_45 = x_64; +x_46 = x_57; x_47 = x_58; x_48 = x_80; goto block_53; @@ -50275,8 +50275,8 @@ else { uint8_t x_81; lean_dec(x_58); +lean_dec(x_57); lean_dec(x_56); -lean_dec(x_55); lean_dec(x_54); x_81 = !lean_is_exclusive(x_63); if (x_81 == 0) @@ -50374,11 +50374,11 @@ x_123 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset___closed__2; x_124 = lean_int_dec_lt(x_123, x_122); if (x_124 == 0) { -x_54 = x_106; -x_55 = x_111; -x_56 = x_120; -x_57 = x_116; -x_58 = x_117; +x_54 = x_120; +x_55 = x_116; +x_56 = x_117; +x_57 = x_106; +x_58 = x_111; x_59 = x_121; goto block_85; } @@ -50398,8 +50398,8 @@ lean_object* x_127; lean_object* x_128; x_127 = lean_nat_abs(x_122); lean_dec(x_122); x_128 = l_Nat_reprFast(x_127); -x_5 = x_121; -x_6 = x_125; +x_5 = x_125; +x_6 = x_121; x_7 = x_128; goto block_13; } @@ -50417,8 +50417,8 @@ lean_dec(x_131); x_134 = l_Nat_reprFast(x_133); x_135 = lean_string_append(x_132, x_134); lean_dec_ref(x_134); -x_5 = x_121; -x_6 = x_125; +x_5 = x_125; +x_6 = x_121; x_7 = x_135; goto block_13; } @@ -50430,11 +50430,11 @@ lean_object* x_136; x_136 = lean_ctor_get(x_119, 0); lean_inc(x_136); lean_dec_ref(x_119); -x_54 = x_106; -x_55 = x_111; -x_56 = x_120; -x_57 = x_116; -x_58 = x_117; +x_54 = x_120; +x_55 = x_116; +x_56 = x_117; +x_57 = x_106; +x_58 = x_111; x_59 = x_136; goto block_85; } @@ -58931,7 +58931,7 @@ return x_4; LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build(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_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_127; lean_object* x_128; uint8_t x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; lean_object* x_143; lean_object* x_144; uint8_t 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_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_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; uint8_t x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_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_228; uint8_t 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; uint8_t x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_251; uint8_t x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_265; uint8_t x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; uint8_t x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; uint8_t x_289; uint8_t 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_305; uint8_t x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_327; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; lean_object* x_143; lean_object* x_144; 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_156; lean_object* x_157; uint8_t 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_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; uint8_t 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_214; 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_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_240; lean_object* x_241; uint8_t 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_251; lean_object* x_252; uint8_t x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_265; lean_object* x_266; uint8_t x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_283; lean_object* x_284; uint8_t x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; uint8_t x_289; lean_object* x_295; uint8_t x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_305; uint8_t x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_327; x_172 = lean_ctor_get(x_1, 0); lean_inc(x_172); x_173 = lean_ctor_get(x_1, 1); @@ -59040,15 +59040,15 @@ goto block_333; block_25: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_7 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_5, 0); lean_inc(x_7); -x_8 = lean_ctor_get(x_3, 1); +x_8 = lean_ctor_get(x_5, 1); lean_inc(x_8); -lean_dec_ref(x_3); +lean_dec_ref(x_5); x_9 = l_Std_Time_TimeZone_LocalTimeType_getTimeZone(x_6); lean_dec_ref(x_6); x_10 = l_Std_Time_TimeZone_toSeconds(x_9); -x_11 = lean_nat_to_int(x_5); +x_11 = lean_nat_to_int(x_3); x_12 = lean_int_neg(x_10); x_13 = lean_int_neg(x_11); lean_dec(x_11); @@ -59090,8 +59090,8 @@ x_30 = lean_ctor_get(x_29, 1); lean_inc_ref(x_30); lean_dec_ref(x_29); x_3 = x_26; -x_4 = x_28; -x_5 = x_27; +x_4 = x_27; +x_5 = x_28; x_6 = x_30; goto block_25; } @@ -59100,8 +59100,8 @@ goto block_25; if (lean_obj_tag(x_2) == 0) { lean_dec_ref(x_35); -lean_dec_ref(x_34); -lean_dec(x_33); +lean_dec(x_34); +lean_dec_ref(x_32); if (lean_obj_tag(x_36) == 0) { lean_object* x_37; @@ -59271,8 +59271,8 @@ if (lean_obj_tag(x_36) == 0) { lean_object* x_100; lean_dec_ref(x_35); -lean_dec_ref(x_34); -lean_dec(x_33); +lean_dec(x_34); +lean_dec_ref(x_32); x_100 = lean_box(0); return x_100; } @@ -59288,10 +59288,10 @@ lean_inc(x_103); x_104 = 0; x_105 = 1; x_106 = lean_alloc_ctor(0, 3, 3); -lean_ctor_set(x_106, 0, x_33); -lean_ctor_set(x_106, 1, x_35); -lean_ctor_set(x_106, 2, x_34); -lean_ctor_set_uint8(x_106, sizeof(void*)*3, x_32); +lean_ctor_set(x_106, 0, x_34); +lean_ctor_set(x_106, 1, x_32); +lean_ctor_set(x_106, 2, x_35); +lean_ctor_set_uint8(x_106, sizeof(void*)*3, x_33); lean_ctor_set_uint8(x_106, sizeof(void*)*3 + 1, x_104); lean_ctor_set_uint8(x_106, sizeof(void*)*3 + 2, x_105); x_107 = lean_unsigned_to_nat(0u); @@ -59330,18 +59330,18 @@ lean_dec(x_103); if (x_123 == 0) { lean_dec(x_117); -x_26 = x_102; -x_27 = x_107; -x_28 = x_109; +x_26 = x_107; +x_27 = x_109; +x_28 = x_102; x_29 = x_113; goto block_31; } else { lean_dec(x_113); -x_26 = x_102; -x_27 = x_107; -x_28 = x_109; +x_26 = x_107; +x_27 = x_109; +x_28 = x_102; x_29 = x_117; goto block_31; } @@ -59354,9 +59354,9 @@ lean_dec(x_103); x_124 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__1; if (lean_obj_tag(x_124) == 0) { -x_3 = x_102; +x_3 = x_107; x_4 = x_109; -x_5 = x_107; +x_5 = x_102; x_6 = x_106; goto block_25; } @@ -59366,9 +59366,9 @@ lean_object* x_125; lean_dec_ref(x_106); x_125 = lean_ctor_get(x_124, 0); lean_inc(x_125); -x_26 = x_102; -x_27 = x_107; -x_28 = x_109; +x_26 = x_107; +x_27 = x_109; +x_28 = x_102; x_29 = x_125; goto block_31; } @@ -59379,21 +59379,21 @@ goto block_31; block_142: { lean_object* x_136; uint8_t x_137; -x_136 = l_Std_Time_Month_Ordinal_days(x_135, x_134); -x_137 = lean_int_dec_le(x_133, x_136); +x_136 = l_Std_Time_Month_Ordinal_days(x_135, x_132); +x_137 = lean_int_dec_le(x_128, x_136); lean_dec(x_136); if (x_137 == 0) { lean_object* x_138; lean_dec(x_134); -lean_dec(x_133); lean_dec(x_132); -lean_dec_ref(x_127); +lean_dec_ref(x_129); +lean_dec(x_128); x_138 = lean_box(0); -x_32 = x_129; -x_33 = x_128; -x_34 = x_130; -x_35 = x_131; +x_32 = x_127; +x_33 = x_130; +x_34 = x_131; +x_35 = x_133; x_36 = x_138; goto block_126; } @@ -59401,18 +59401,18 @@ else { lean_object* x_139; lean_object* x_140; lean_object* x_141; x_139 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_139, 0, x_132); -lean_ctor_set(x_139, 1, x_134); -lean_ctor_set(x_139, 2, x_133); +lean_ctor_set(x_139, 0, x_134); +lean_ctor_set(x_139, 1, x_132); +lean_ctor_set(x_139, 2, x_128); x_140 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_127); +lean_ctor_set(x_140, 1, x_129); x_141 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_141, 0, x_140); -x_32 = x_129; -x_33 = x_128; -x_34 = x_130; -x_35 = x_131; +x_32 = x_127; +x_33 = x_130; +x_34 = x_131; +x_35 = x_133; x_36 = x_141; goto block_126; } @@ -59421,9 +59421,9 @@ goto block_126; { lean_object* x_152; lean_object* x_153; uint8_t x_154; x_152 = l___private_Std_Time_Format_Basic_0__Std_Time_dateFromModifier___closed__1; -x_153 = lean_int_mod(x_149, x_152); -x_154 = lean_int_dec_eq(x_153, x_147); -lean_dec(x_147); +x_153 = lean_int_mod(x_151, x_152); +x_154 = lean_int_dec_eq(x_153, x_148); +lean_dec(x_148); lean_dec(x_153); if (x_154 == 0) { @@ -59431,11 +59431,11 @@ x_127 = x_143; x_128 = x_144; x_129 = x_145; x_130 = x_146; -x_131 = x_148; +x_131 = x_147; x_132 = x_149; -x_133 = x_151; -x_134 = x_150; -x_135 = x_145; +x_133 = x_150; +x_134 = x_151; +x_135 = x_146; goto block_142; } else @@ -59444,10 +59444,10 @@ x_127 = x_143; x_128 = x_144; x_129 = x_145; x_130 = x_146; -x_131 = x_148; +x_131 = x_147; x_132 = x_149; -x_133 = x_151; -x_134 = x_150; +x_133 = x_150; +x_134 = x_151; x_135 = x_154; goto block_142; } @@ -59456,40 +59456,40 @@ goto block_142; { lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; x_164 = l___private_Std_Time_Format_Basic_0__Std_Time_dateFromModifier___closed__0; -x_165 = lean_int_mod(x_160, x_164); +x_165 = lean_int_mod(x_162, x_164); x_166 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; x_167 = lean_int_dec_eq(x_165, x_166); lean_dec(x_165); if (x_167 == 0) { -x_127 = x_163; +x_127 = x_156; x_128 = x_157; -x_129 = x_156; +x_129 = x_163; x_130 = x_158; x_131 = x_159; x_132 = x_160; -x_133 = x_162; -x_134 = x_161; -x_135 = x_156; +x_133 = x_161; +x_134 = x_162; +x_135 = x_158; goto block_142; } else { lean_object* x_168; lean_object* x_169; uint8_t x_170; x_168 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__0; -x_169 = lean_int_mod(x_160, x_168); +x_169 = lean_int_mod(x_162, x_168); x_170 = lean_int_dec_eq(x_169, x_166); lean_dec(x_169); if (x_170 == 0) { if (x_167 == 0) { -x_143 = x_163; +x_143 = x_156; x_144 = x_157; -x_145 = x_156; +x_145 = x_163; x_146 = x_158; -x_147 = x_166; -x_148 = x_159; +x_147 = x_159; +x_148 = x_166; x_149 = x_160; x_150 = x_161; x_151 = x_162; @@ -59497,26 +59497,26 @@ goto block_155; } else { -x_127 = x_163; +x_127 = x_156; x_128 = x_157; -x_129 = x_156; +x_129 = x_163; x_130 = x_158; x_131 = x_159; x_132 = x_160; -x_133 = x_162; -x_134 = x_161; +x_133 = x_161; +x_134 = x_162; x_135 = x_167; goto block_142; } } else { -x_143 = x_163; +x_143 = x_156; x_144 = x_157; -x_145 = x_156; +x_145 = x_163; x_146 = x_158; -x_147 = x_166; -x_148 = x_159; +x_147 = x_159; +x_148 = x_166; x_149 = x_160; x_150 = x_161; x_151 = x_162; @@ -59532,16 +59532,16 @@ if (lean_obj_tag(x_185) == 0) { lean_object* x_206; x_206 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_206, 0, x_198); -lean_ctor_set(x_206, 1, x_200); -lean_ctor_set(x_206, 2, x_195); +lean_ctor_set(x_206, 0, x_204); +lean_ctor_set(x_206, 1, x_199); +lean_ctor_set(x_206, 2, x_196); lean_ctor_set(x_206, 3, x_205); -x_156 = x_197; -x_157 = x_196; -x_158 = x_199; -x_159 = x_201; -x_160 = x_202; -x_161 = x_204; +x_156 = x_195; +x_157 = x_197; +x_158 = x_198; +x_159 = x_200; +x_160 = x_201; +x_161 = x_202; x_162 = x_203; x_163 = x_206; goto block_171; @@ -59550,9 +59550,9 @@ else { lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_dec(x_205); -lean_dec(x_200); -lean_dec(x_198); -lean_dec(x_195); +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_196); x_207 = lean_ctor_get(x_185, 0); lean_inc(x_207); lean_dec_ref(x_185); @@ -59561,12 +59561,12 @@ x_209 = lean_int_mul(x_207, x_208); lean_dec(x_207); x_210 = l_Std_Time_PlainTime_ofNanoseconds(x_209); lean_dec(x_209); -x_156 = x_197; -x_157 = x_196; -x_158 = x_199; -x_159 = x_201; -x_160 = x_202; -x_161 = x_204; +x_156 = x_195; +x_157 = x_197; +x_158 = x_198; +x_159 = x_200; +x_160 = x_201; +x_161 = x_202; x_162 = x_203; x_163 = x_210; goto block_171; @@ -59576,21 +59576,21 @@ else { lean_object* x_211; lean_object* x_212; lean_dec(x_205); -lean_dec(x_200); -lean_dec(x_198); -lean_dec(x_195); +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_196); lean_dec(x_185); x_211 = lean_ctor_get(x_187, 0); lean_inc(x_211); lean_dec_ref(x_187); x_212 = l_Std_Time_PlainTime_ofNanoseconds(x_211); lean_dec(x_211); -x_156 = x_197; -x_157 = x_196; -x_158 = x_199; -x_159 = x_201; -x_160 = x_202; -x_161 = x_204; +x_156 = x_195; +x_157 = x_197; +x_158 = x_198; +x_159 = x_200; +x_160 = x_201; +x_161 = x_202; x_162 = x_203; x_163 = x_212; goto block_171; @@ -59604,12 +59604,12 @@ if (lean_obj_tag(x_184) == 0) { lean_object* x_224; x_224 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__4; -x_195 = x_223; -x_196 = x_215; -x_197 = x_214; +x_195 = x_214; +x_196 = x_223; +x_197 = x_215; x_198 = x_216; -x_199 = x_218; -x_200 = x_217; +x_199 = x_217; +x_200 = x_218; x_201 = x_219; x_202 = x_220; x_203 = x_222; @@ -59623,12 +59623,12 @@ lean_object* x_225; x_225 = lean_ctor_get(x_184, 0); lean_inc(x_225); lean_dec_ref(x_184); -x_195 = x_223; -x_196 = x_215; -x_197 = x_214; +x_195 = x_214; +x_196 = x_223; +x_197 = x_215; x_198 = x_216; -x_199 = x_218; -x_200 = x_217; +x_199 = x_217; +x_200 = x_218; x_201 = x_219; x_202 = x_220; x_203 = x_222; @@ -59644,12 +59644,12 @@ lean_dec(x_184); x_226 = lean_ctor_get(x_186, 0); lean_inc(x_226); lean_dec_ref(x_186); -x_195 = x_223; -x_196 = x_215; -x_197 = x_214; +x_195 = x_214; +x_196 = x_223; +x_197 = x_215; x_198 = x_216; -x_199 = x_218; -x_200 = x_217; +x_199 = x_217; +x_200 = x_218; x_201 = x_219; x_202 = x_220; x_203 = x_222; @@ -59664,8 +59664,8 @@ if (lean_obj_tag(x_183) == 0) { lean_object* x_237; x_237 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__5; -x_214 = x_229; -x_215 = x_228; +x_214 = x_228; +x_215 = x_229; x_216 = x_230; x_217 = x_236; x_218 = x_231; @@ -59682,8 +59682,8 @@ lean_object* x_238; x_238 = lean_ctor_get(x_183, 0); lean_inc(x_238); lean_dec_ref(x_183); -x_214 = x_229; -x_215 = x_228; +x_214 = x_228; +x_215 = x_229; x_216 = x_230; x_217 = x_236; x_218 = x_231; @@ -59701,14 +59701,14 @@ if (lean_obj_tag(x_182) == 0) { lean_object* x_248; x_248 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__13; -x_228 = x_241; -x_229 = x_240; -x_230 = x_247; -x_231 = x_242; -x_232 = x_243; -x_233 = x_244; +x_228 = x_240; +x_229 = x_241; +x_230 = x_242; +x_231 = x_243; +x_232 = x_244; +x_233 = x_245; x_234 = x_246; -x_235 = x_245; +x_235 = x_247; x_236 = x_248; goto block_239; } @@ -59718,14 +59718,14 @@ lean_object* x_249; x_249 = lean_ctor_get(x_182, 0); lean_inc(x_249); lean_dec_ref(x_182); -x_228 = x_241; -x_229 = x_240; -x_230 = x_247; -x_231 = x_242; -x_232 = x_243; -x_233 = x_244; +x_228 = x_240; +x_229 = x_241; +x_230 = x_242; +x_231 = x_243; +x_232 = x_244; +x_233 = x_245; x_234 = x_246; -x_235 = x_245; +x_235 = x_247; x_236 = x_249; goto block_239; } @@ -59738,13 +59738,13 @@ if (lean_obj_tag(x_181) == 0) { lean_object* x_258; x_258 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; -x_240 = x_252; -x_241 = x_251; +x_240 = x_251; +x_241 = x_252; x_242 = x_253; x_243 = x_254; x_244 = x_255; -x_245 = x_257; -x_246 = x_256; +x_245 = x_256; +x_246 = x_257; x_247 = x_258; goto block_250; } @@ -59754,13 +59754,13 @@ lean_object* x_259; x_259 = lean_ctor_get(x_181, 0); lean_inc(x_259); lean_dec_ref(x_181); -x_240 = x_252; -x_241 = x_251; +x_240 = x_251; +x_241 = x_252; x_242 = x_253; x_243 = x_254; x_244 = x_255; -x_245 = x_257; -x_246 = x_256; +x_245 = x_256; +x_246 = x_257; x_247 = x_259; goto block_250; } @@ -59776,13 +59776,13 @@ lean_dec_ref(x_180); x_261 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset___closed__13; x_262 = lean_int_add(x_260, x_261); lean_dec(x_260); -x_240 = x_252; -x_241 = x_251; +x_240 = x_251; +x_241 = x_252; x_242 = x_253; x_243 = x_254; x_244 = x_255; -x_245 = x_257; -x_246 = x_256; +x_245 = x_256; +x_246 = x_257; x_247 = x_262; goto block_250; } @@ -59793,13 +59793,13 @@ lean_dec_ref(x_180); x_263 = lean_ctor_get(x_181, 0); lean_inc(x_263); lean_dec_ref(x_181); -x_240 = x_252; -x_241 = x_251; +x_240 = x_251; +x_241 = x_252; x_242 = x_253; x_243 = x_254; x_244 = x_255; -x_245 = x_257; -x_246 = x_256; +x_245 = x_256; +x_246 = x_257; x_247 = x_263; goto block_250; } @@ -59818,9 +59818,9 @@ x_251 = x_265; x_252 = x_266; x_253 = x_267; x_254 = x_268; -x_255 = x_271; -x_256 = x_269; -x_257 = x_270; +x_255 = x_269; +x_256 = x_270; +x_257 = x_271; goto block_264; } else @@ -59841,13 +59841,13 @@ x_276 = lean_unbox(x_272); lean_dec(x_272); x_277 = l_Std_Time_HourMarker_toAbsolute(x_276, x_275); lean_dec(x_275); -x_240 = x_266; -x_241 = x_265; +x_240 = x_265; +x_241 = x_266; x_242 = x_267; x_243 = x_268; -x_244 = x_271; +x_244 = x_269; x_245 = x_270; -x_246 = x_269; +x_246 = x_271; x_247 = x_277; goto block_250; } @@ -59868,13 +59868,13 @@ x_280 = lean_unbox(x_278); lean_dec(x_278); x_281 = l_Std_Time_HourMarker_toAbsolute(x_280, x_279); lean_dec(x_279); -x_240 = x_266; -x_241 = x_265; +x_240 = x_265; +x_241 = x_266; x_242 = x_267; x_243 = x_268; -x_244 = x_271; +x_244 = x_269; x_245 = x_270; -x_246 = x_269; +x_246 = x_271; x_247 = x_281; goto block_250; } @@ -59888,9 +59888,9 @@ x_251 = x_265; x_252 = x_266; x_253 = x_267; x_254 = x_268; -x_255 = x_271; -x_256 = x_269; -x_257 = x_270; +x_255 = x_269; +x_256 = x_270; +x_257 = x_271; goto block_264; } } @@ -59902,12 +59902,12 @@ if (lean_obj_tag(x_173) == 0) { lean_object* x_290; x_290 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__0; -x_265 = x_284; -x_266 = x_283; +x_265 = x_283; +x_266 = x_284; x_267 = x_285; x_268 = x_286; -x_269 = x_288; -x_270 = x_287; +x_269 = x_287; +x_270 = x_288; x_271 = x_290; goto block_282; } @@ -59919,12 +59919,12 @@ lean_inc(x_291); lean_dec_ref(x_173); x_292 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_convertYearAndEra(x_291, x_289); lean_dec(x_291); -x_265 = x_284; -x_266 = x_283; +x_265 = x_283; +x_266 = x_284; x_267 = x_285; x_268 = x_286; -x_269 = x_288; -x_270 = x_287; +x_269 = x_287; +x_270 = x_288; x_271 = x_292; goto block_282; } @@ -59936,12 +59936,12 @@ lean_dec(x_173); x_293 = lean_ctor_get(x_174, 0); lean_inc(x_293); lean_dec_ref(x_174); -x_265 = x_284; -x_266 = x_283; +x_265 = x_283; +x_266 = x_284; x_267 = x_285; x_268 = x_286; -x_269 = x_288; -x_270 = x_287; +x_269 = x_287; +x_270 = x_288; x_271 = x_293; goto block_282; } @@ -59953,11 +59953,11 @@ if (lean_obj_tag(x_172) == 0) uint8_t x_301; x_301 = 1; x_283 = x_295; -x_284 = x_296; -x_285 = x_297; -x_286 = x_298; -x_287 = x_299; -x_288 = x_300; +x_284 = x_300; +x_285 = x_296; +x_286 = x_297; +x_287 = x_298; +x_288 = x_299; x_289 = x_301; goto block_294; } @@ -59970,11 +59970,11 @@ lean_dec_ref(x_172); x_303 = lean_unbox(x_302); lean_dec(x_302); x_283 = x_295; -x_284 = x_296; -x_285 = x_297; -x_286 = x_298; -x_287 = x_299; -x_288 = x_300; +x_284 = x_300; +x_285 = x_296; +x_286 = x_297; +x_287 = x_298; +x_288 = x_299; x_289 = x_303; goto block_294; } @@ -59985,11 +59985,11 @@ if (lean_obj_tag(x_176) == 0) { lean_object* x_310; x_310 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__22; -x_295 = x_306; -x_296 = x_305; +x_295 = x_305; +x_296 = x_306; x_297 = x_307; -x_298 = x_308; -x_299 = x_309; +x_298 = x_309; +x_299 = x_308; x_300 = x_310; goto block_304; } @@ -59999,11 +59999,11 @@ lean_object* x_311; x_311 = lean_ctor_get(x_176, 0); lean_inc(x_311); lean_dec_ref(x_176); -x_295 = x_306; -x_296 = x_305; +x_295 = x_305; +x_296 = x_306; x_297 = x_307; -x_298 = x_308; -x_299 = x_309; +x_298 = x_309; +x_299 = x_308; x_300 = x_311; goto block_304; } @@ -60016,10 +60016,10 @@ if (lean_obj_tag(x_175) == 0) { lean_object* x_317; x_317 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__29; -x_305 = x_313; +x_305 = x_315; x_306 = x_316; -x_307 = x_314; -x_308 = x_315; +x_307 = x_313; +x_308 = x_314; x_309 = x_317; goto block_312; } @@ -60029,10 +60029,10 @@ lean_object* x_318; x_318 = lean_ctor_get(x_175, 0); lean_inc(x_318); lean_dec_ref(x_175); -x_305 = x_313; +x_305 = x_315; x_306 = x_316; -x_307 = x_314; -x_308 = x_315; +x_307 = x_313; +x_308 = x_314; x_309 = x_318; goto block_312; } From c050b3a3a70a86430ffd4409f55afd484dbbe278 Mon Sep 17 00:00:00 2001 From: Sebastian Ullrich Date: Wed, 24 Dec 2025 11:55:32 +0000 Subject: [PATCH 3/5] feat: `@[allow_native_decide]` kernel check --- src/Lean/AllowNativeDecide.lean | 18 ++++++++++++++++++ src/kernel/type_checker.cpp | 9 +++++++++ 2 files changed, 27 insertions(+) diff --git a/src/Lean/AllowNativeDecide.lean b/src/Lean/AllowNativeDecide.lean index d09133b1314b..d639de6a25a9 100644 --- a/src/Lean/AllowNativeDecide.lean +++ b/src/Lean/AllowNativeDecide.lean @@ -14,3 +14,21 @@ namespace Lean builtin_initialize allowNativeDecideAttr : TagAttribute ← registerTagAttribute `allow_native_decide "mark definition as allowed to be used in `native_decide` computations" + +@[export lean_has_disallowed_native_decide] +partial def hasDisallowedNativeDecide (kenv : Kernel.Environment) (n : Name) : Option Name := + let env := Environment.ofKernelEnv kenv + go env n +where go (env : Environment) (n : Name) : Option Name := Id.run do + let some c := kenv.find? n | return some n + match c with + | .defnInfo d => + if allowNativeDecideAttr.hasTag env d.name then + none + else if !n.isInternalDetail then + some n + else + return d.value.foldConsts (init := none) (go env · <|> ·) + | .ctorInfo _ => none + | .inductInfo _ => none + | c => some c.name diff --git a/src/kernel/type_checker.cpp b/src/kernel/type_checker.cpp index 2f681e45af4d..e4234e434d50 100644 --- a/src/kernel/type_checker.cpp +++ b/src/kernel/type_checker.cpp @@ -9,6 +9,7 @@ Author: Leonardo de Moura #include "runtime/interrupt.h" #include "runtime/sstream.h" #include "runtime/flet.h" +#include "runtime/option_ref.h" #include "util/lbool.h" #include "kernel/type_checker.h" #include "kernel/expr_maps.h" @@ -534,11 +535,16 @@ object * run_boxed_kernel(environment const & env, options const & opts, name co expr mk_bool_true(); expr mk_bool_false(); +extern "C" object * lean_has_disallowed_native_decide(object * env, object * n); + optional reduce_native(environment const & env, expr const & e) { if (!is_app(e)) return none_expr(); expr const & arg = app_arg(e); if (!is_constant(arg)) return none_expr(); if (app_fn(e) == *g_lean_reduce_bool) { + if (option_ref has_disallowed = option_ref(lean_has_disallowed_native_decide(env.to_obj_arg(), const_name(arg).to_obj_arg()))) { + throw kernel_exception(env, sstream() << "cannot native-reduce expression involving definition `" << has_disallowed.get_val() << "` not marked `@[allow_native_decide]`"); + } object * r = ir::run_boxed_kernel(env, options(), const_name(arg), 0, nullptr); if (!lean_is_scalar(r)) { lean_dec_ref(r); @@ -547,6 +553,9 @@ optional reduce_native(environment const & env, expr const & e) { return lean_unbox(r) == 0 ? some_expr(mk_bool_false()) : some_expr(mk_bool_true()); } if (app_fn(e) == *g_lean_reduce_nat) { + if (option_ref has_disallowed = option_ref(lean_has_disallowed_native_decide(env.to_obj_arg(), const_name(arg).to_obj_arg()))) { + throw kernel_exception(env, sstream() << "cannot native-reduce expression involving definition `" << has_disallowed.get_val() << "` not marked `@[allow_native_decide]`"); + } object * r = ir::run_boxed_kernel(env, options(), const_name(arg), 0, nullptr); if (lean_is_scalar(r) || lean_is_mpz(r)) { return some_expr(mk_lit(literal(nat(r)))); From 26dea2d928c1ce6739845dc5dcd201687ebd9ca1 Mon Sep 17 00:00:00 2001 From: Sebastian Ullrich Date: Wed, 24 Dec 2025 11:55:32 +0000 Subject: [PATCH 4/5] feat: add `@[allow_native_decide]` annotations for `bv_decide` --- src/Init/Prelude.lean | 8 +++++--- src/Std/Tactic/BVDecide/Reflect.lean | 2 +- 2 files changed, 6 insertions(+), 4 deletions(-) diff --git a/src/Init/Prelude.lean b/src/Init/Prelude.lean index cdba6731bfca..3bbf7c4ea420 100644 --- a/src/Init/Prelude.lean +++ b/src/Init/Prelude.lean @@ -1019,7 +1019,7 @@ support. | true, false => isFalse (fun h => Bool.noConfusion h) | true, true => isTrue rfl -@[inline] instance : DecidableEq Bool := +@[inline, allow_native_decide] instance : DecidableEq Bool := Bool.decEq /-- @@ -1236,7 +1236,9 @@ class OfNat (α : Type u) (_ : Nat) where `α`. -/ ofNat : α -@[default_instance 100] /- low prio -/ +attribute [allow_native_decide] OfNat.ofNat + +@[default_instance 100, allow_native_decide] /- low prio -/ instance instOfNatNat (n : Nat) : OfNat Nat n where ofNat := n @@ -2354,7 +2356,7 @@ protected def BitVec.ofNatLT {w : Nat} (i : Nat) (p : LT.lt i (hPow 2 w)) : BitV /-- The bitvector with value `i mod 2^n`. -/ -@[expose, match_pattern] +@[expose, match_pattern, allow_native_decide] protected def BitVec.ofNat (n : Nat) (i : Nat) : BitVec n where toFin := Fin.Internal.ofNat (HPow.hPow 2 n) (Nat.pow_pos (Nat.zero_lt_succ _)) i diff --git a/src/Std/Tactic/BVDecide/Reflect.lean b/src/Std/Tactic/BVDecide/Reflect.lean index 4f175d9d73cc..0965aebb0d0f 100644 --- a/src/Std/Tactic/BVDecide/Reflect.lean +++ b/src/Std/Tactic/BVDecide/Reflect.lean @@ -183,7 +183,7 @@ theorem verifyCert_correct : ∀ cnf cert, verifyCert cnf cert = true → cnf.Un /-- Verify that `cert` is an UNSAT proof for the SAT problem obtained by bitblasting `bv`. -/ -def verifyBVExpr (bv : BVLogicalExpr) (cert : String) : Bool := +@[allow_native_decide] def verifyBVExpr (bv : BVLogicalExpr) (cert : String) : Bool := verifyCert (AIG.toCNF bv.bitblast.relabelNat) cert theorem unsat_of_verifyBVExpr_eq_true (bv : BVLogicalExpr) (c : String) From 3276dbd622bf220e43c0b7759f71043a1a9f0da6 Mon Sep 17 00:00:00 2001 From: Sebastian Ullrich Date: Wed, 24 Dec 2025 11:55:32 +0000 Subject: [PATCH 5/5] chore: remove uses of `native_decide` in core, should be `#eval` tests --- src/Lean/Data/Lsp/LanguageFeatures.lean | 10 ---------- src/lake/Lake/Build/Trace.lean | 4 ---- 2 files changed, 14 deletions(-) diff --git a/src/Lean/Data/Lsp/LanguageFeatures.lean b/src/Lean/Data/Lsp/LanguageFeatures.lean index 562d97109be4..a20bf64b40fb 100644 --- a/src/Lean/Data/Lsp/LanguageFeatures.lean +++ b/src/Lean/Data/Lsp/LanguageFeatures.lean @@ -465,11 +465,6 @@ def SemanticTokenType.names : Array String := def SemanticTokenType.toNat (tokenType : SemanticTokenType) : Nat := tokenType.ctorIdx --- sanity check -example {v : SemanticTokenType} : open SemanticTokenType in - names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by - cases v <;> native_decide - /-- The semantic token modifiers included by default in the LSP specification. Not used by the Lean core, but implementing them here allows them to be @@ -496,11 +491,6 @@ def SemanticTokenModifier.names : Array String := def SemanticTokenModifier.toNat (modifier : SemanticTokenModifier) : Nat := modifier.ctorIdx --- sanity check -example {v : SemanticTokenModifier} : open SemanticTokenModifier in - names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by - cases v <;> native_decide - structure SemanticTokensLegend where tokenTypes : Array String tokenModifiers : Array String diff --git a/src/lake/Lake/Build/Trace.lean b/src/lake/Lake/Build/Trace.lean index f7e775b8653f..7666183a1236 100644 --- a/src/lake/Lake/Build/Trace.lean +++ b/src/lake/Lake/Build/Trace.lean @@ -130,10 +130,6 @@ public def ofHex (s : String) : Hash := else if 97 ≤ c then n*16 + (c - 87).toUInt64 -- c - 'a' + 10 = (c - 87) else n*16 + (c - 55).toUInt64 -- c - 'A' + 10 = (c - 55) --- sanity check -example : ofHex "0123456789" = ⟨0x0123456789⟩ ∧ - ofHex "abcdeF" = ⟨0xabcdef⟩ ∧ ofHex "ABCDEF" = ⟨0xABCDEF⟩ := by native_decide - /-- Parse a hash from a 16-digit string of hexadecimal digits. -/ public def ofHex? (s : String) : Option Hash := if s.utf8ByteSize = 16 && isHex s then ofHex s else none