diff --git a/.github/workflows/ci.yml b/.github/workflows/ci.yml index 861f7349a2b6..a2433a217fee 100644 --- a/.github/workflows/ci.yml +++ b/.github/workflows/ci.yml @@ -216,7 +216,7 @@ jobs: brew install ccache tree zstd coreutils gmp if: matrix.os == 'macos-latest' - name: Setup emsdk - uses: mymindstorm/setup-emsdk@v11 + uses: mymindstorm/setup-emsdk@v12 with: version: 3.1.44 actions-cache-folder: emsdk diff --git a/RELEASES.md b/RELEASES.md index 02c510ecace9..c880e2a3fecf 100644 --- a/RELEASES.md +++ b/RELEASES.md @@ -11,6 +11,8 @@ of each version. v4.4.0 (development in progress) --------- +* By default, `simp` will no longer try to use Decidable instances to rewrite terms. In particular, not all decidable goals will be closed by `simp`, and the `decide` tactic may be useful in such cases. The `decide` simp configuration option can be used to locally restore the old `simp` behavior, as in `simp (config := {decide := true})`; this includes using Decidable instances to verify side goals such as numeric inequalities. + v4.3.0 --------- diff --git a/src/Init/Data/Nat/Basic.lean b/src/Init/Data/Nat/Basic.lean index e3c811420295..707a383d96f4 100644 --- a/src/Init/Data/Nat/Basic.lean +++ b/src/Init/Data/Nat/Basic.lean @@ -629,7 +629,7 @@ protected theorem sub_lt_sub_left : ∀ {k m n : Nat}, k < m → k < n → m - n @[simp] protected theorem zero_sub (n : Nat) : 0 - n = 0 := by induction n with | zero => rfl - | succ n ih => simp [ih, Nat.sub_succ] + | succ n ih => simp only [ih, Nat.sub_succ]; decide protected theorem sub_self_add (n m : Nat) : n - (n + m) = 0 := by show (n + 0) - (n + m) = 0 diff --git a/src/Init/Meta.lean b/src/Init/Meta.lean index 2f775a6c0584..8088dc202355 100644 --- a/src/Init/Meta.lean +++ b/src/Init/Meta.lean @@ -1252,14 +1252,14 @@ This will rewrite with all equation lemmas, which can be used to partially evaluate many definitions. -/ declare_simp_like_tactic simpAutoUnfold "simp! " fun (c : Lean.Meta.Simp.Config) => { c with autoUnfold := true } -/-- `simp_arith` is shorthand for `simp` with `arith := true`. +/-- `simp_arith` is shorthand for `simp` with `arith := true` and `decide := true`. This enables the use of normalization by linear arithmetic. -/ -declare_simp_like_tactic simpArith "simp_arith " fun (c : Lean.Meta.Simp.Config) => { c with arith := true } +declare_simp_like_tactic simpArith "simp_arith " fun (c : Lean.Meta.Simp.Config) => { c with arith := true, decide := true } /-- `simp_arith!` is shorthand for `simp_arith` with `autoUnfold := true`. This will rewrite with all equation lemmas, which can be used to partially evaluate many definitions. -/ -declare_simp_like_tactic simpArithAutoUnfold "simp_arith! " fun (c : Lean.Meta.Simp.Config) => { c with arith := true, autoUnfold := true } +declare_simp_like_tactic simpArithAutoUnfold "simp_arith! " fun (c : Lean.Meta.Simp.Config) => { c with arith := true, autoUnfold := true, decide := true } /-- `simp_all!` is shorthand for `simp_all` with `autoUnfold := true`. This will rewrite with all equation lemmas, which can be used to @@ -1267,10 +1267,10 @@ partially evaluate many definitions. -/ declare_simp_like_tactic (all := true) simpAllAutoUnfold "simp_all! " fun (c : Lean.Meta.Simp.ConfigCtx) => { c with autoUnfold := true } /-- `simp_all_arith` combines the effects of `simp_all` and `simp_arith`. -/ -declare_simp_like_tactic (all := true) simpAllArith "simp_all_arith " fun (c : Lean.Meta.Simp.ConfigCtx) => { c with arith := true } +declare_simp_like_tactic (all := true) simpAllArith "simp_all_arith " fun (c : Lean.Meta.Simp.ConfigCtx) => { c with arith := true, decide := true } /-- `simp_all_arith!` combines the effects of `simp_all`, `simp_arith` and `simp!`. -/ -declare_simp_like_tactic (all := true) simpAllArithAutoUnfold "simp_all_arith! " fun (c : Lean.Meta.Simp.ConfigCtx) => { c with arith := true, autoUnfold := true } +declare_simp_like_tactic (all := true) simpAllArithAutoUnfold "simp_all_arith! " fun (c : Lean.Meta.Simp.ConfigCtx) => { c with arith := true, autoUnfold := true, decide := true } /-- `dsimp!` is shorthand for `dsimp` with `autoUnfold := true`. This will rewrite with all equation lemmas, which can be used to diff --git a/src/Init/MetaTypes.lean b/src/Init/MetaTypes.lean index d00e5d86293a..2c5a49524e40 100644 --- a/src/Init/MetaTypes.lean +++ b/src/Init/MetaTypes.lean @@ -70,7 +70,7 @@ structure Config where etaStruct : EtaStructMode := .all iota : Bool := true proj : Bool := true - decide : Bool := true + decide : Bool := false arith : Bool := false autoUnfold : Bool := false /-- diff --git a/src/Init/SimpLemmas.lean b/src/Init/SimpLemmas.lean index e8da7cab2a6a..8e11689814da 100644 --- a/src/Init/SimpLemmas.lean +++ b/src/Init/SimpLemmas.lean @@ -104,6 +104,7 @@ theorem dite_congr {_ : Decidable b} [Decidable c] @[simp] theorem implies_true (α : Sort u) : (α → True) = True := eq_true fun _ => trivial @[simp] theorem true_implies (p : Prop) : (True → p) = p := propext ⟨(· trivial), (fun _ => ·)⟩ @[simp] theorem not_false_eq_true : (¬ False) = True := eq_true False.elim +@[simp] theorem not_true_eq_false : (¬ True) = False := by decide @[simp] theorem Bool.or_false (b : Bool) : (b || false) = b := by cases b <;> rfl @[simp] theorem Bool.or_true (b : Bool) : (b || true) = true := by cases b <;> rfl @@ -158,7 +159,7 @@ theorem Bool.or_assoc (a b c : Bool) : (a || b || c) = (a || (b || c)) := by @[simp] theorem bne_self_eq_false' [DecidableEq α] (a : α) : (a != a) = false := by simp [bne] @[simp] theorem Nat.le_zero_eq (a : Nat) : (a ≤ 0) = (a = 0) := - propext ⟨fun h => Nat.le_antisymm h (Nat.zero_le ..), fun h => by simp [h]⟩ + propext ⟨fun h => Nat.le_antisymm h (Nat.zero_le ..), fun h => by rw [h]; decide⟩ @[simp] theorem decide_False : decide False = false := rfl @[simp] theorem decide_True : decide True = true := rfl diff --git a/src/Lean/Compiler/LCNF/PassManager.lean b/src/Lean/Compiler/LCNF/PassManager.lean index 7347e3792aad..66d1d596f474 100644 --- a/src/Lean/Compiler/LCNF/PassManager.lean +++ b/src/Lean/Compiler/LCNF/PassManager.lean @@ -46,7 +46,7 @@ structure Pass where Resulting phase. -/ phaseOut : Phase := phase - phaseInv : phaseOut ≥ phase := by simp + phaseInv : phaseOut ≥ phase := by simp_arith /-- The name of the `Pass` -/ diff --git a/stage0/stdlib/Init/Data/Array/Mem.c b/stage0/stdlib/Init/Data/Array/Mem.c index 212cc0b44a38..62ae5b4bcdcb 100644 --- a/stage0/stdlib/Init/Data/Array/Mem.c +++ b/stage0/stdlib/Init/Data/Array/Mem.c @@ -14,7 +14,11 @@ extern "C" { #endif LEAN_EXPORT lean_object* l___private_Init_Data_Array_Mem_0__List_get_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_tacticArray__mem__dec___closed__1; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__42; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3; +LEAN_EXPORT lean_object* l_Array_tacticArray__mem__dec; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__35; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__25; @@ -23,70 +27,98 @@ static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__tacti static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__3; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__24; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__38; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__9; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__15; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__19; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__26; +lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__11; static lean_object* l_Array_tacticArray__get__dec___closed__4; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__28; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__40; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__27; -LEAN_EXPORT lean_object* l_Array_instMembershipArray___boxed(lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__1; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__10; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Mem_0__List_get_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__44; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__34; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__29; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__13; LEAN_EXPORT lean_object* l_Array_tacticArray__get__dec; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__5; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_tacticArray__get__dec___closed__5; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20; static lean_object* l_Array_tacticArray__get__dec___closed__3; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__14; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__33; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Array_tacticArray__mem__dec___closed__5; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__7; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__30; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1; static lean_object* l_Array_tacticArray__get__dec___closed__6; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__12; +lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__21; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__8; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__41; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Mem_0__List_get_match__1_splitter(lean_object*, lean_object*); +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__36; static lean_object* l_Array_tacticArray__get__dec___closed__1; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__32; +static lean_object* l_Array_tacticArray__mem__dec___closed__4; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__31; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__18; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__6; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_instMembershipArray(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_instMembershipArray(lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__20; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__22; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__37; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__4; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Array_tacticArray__mem__dec___closed__2; LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_tacticArray__get__dec___closed__2; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__16; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__17; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__23; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13; +static lean_object* l_Array_tacticArray__mem__dec___closed__3; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__39; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10; LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1(lean_object*, lean_object*, lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21; LEAN_EXPORT lean_object* l___private_Init_Data_Array_Mem_0__List_get_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -133,21 +165,12 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Array_instMembershipArray(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_instMembershipArray(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_instMembershipArray___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Array_instMembershipArray(x_1, x_2); -lean_dec(x_2); -return x_3; +lean_object* x_2; +x_2 = lean_box(0); +return x_2; } } static lean_object* _init_l_Array_tacticArray__get__dec___closed__1() { @@ -841,6 +864,538 @@ return x_15; } } } +static lean_object* _init_l_Array_tacticArray__mem__dec___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tacticArray_mem_dec", 19); +return x_1; +} +} +static lean_object* _init_l_Array_tacticArray__mem__dec___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_tacticArray__get__dec___closed__1; +x_2 = l_Array_tacticArray__mem__dec___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array_tacticArray__mem__dec___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("array_mem_dec", 13); +return x_1; +} +} +static lean_object* _init_l_Array_tacticArray__mem__dec___closed__4() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; +x_1 = l_Array_tacticArray__mem__dec___closed__3; +x_2 = 0; +x_3 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array_tacticArray__mem__dec___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Array_tacticArray__mem__dec___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Array_tacticArray__mem__dec___closed__4; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Array_tacticArray__mem__dec() { +_start: +{ +lean_object* x_1; +x_1 = l_Array_tacticArray__mem__dec___closed__5; +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Array.sizeOf_lt_of_mem", 22); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("sizeOf_lt_of_mem", 16); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_tacticArray__get__dec___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("assumption", 10); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +x_3 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__3; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("done", 4); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +x_3 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__3; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("syntheticHole", 13); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +x_3 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__23; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("?", 1); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("h", 1); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("case'", 5); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +x_3 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__3; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("caseArg", 7); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; +x_3 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__3; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("binderIdent", 11); +return x_1; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; +x_2 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("=>", 2); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Array_tacticArray__mem__dec___closed__2; +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; 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; +x_8 = lean_ctor_get(x_2, 5); +lean_inc(x_8); +x_9 = 0; +x_10 = l_Lean_SourceInfo_fromRef(x_8, x_9); +x_11 = lean_ctor_get(x_2, 2); +lean_inc(x_11); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +lean_dec(x_2); +x_13 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__4; +lean_inc(x_10); +x_14 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_14, 0, x_10); +lean_ctor_set(x_14, 1, x_13); +x_15 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__10; +lean_inc(x_10); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_10); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__15; +lean_inc(x_10); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_10); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4; +lean_inc(x_11); +lean_inc(x_12); +x_20 = l_Lean_addMacroScope(x_12, x_19, x_11); +x_21 = lean_box(0); +x_22 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2; +x_23 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6; +lean_inc(x_10); +x_24 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_24, 0, x_10); +lean_ctor_set(x_24, 1, x_22); +lean_ctor_set(x_24, 2, x_20); +lean_ctor_set(x_24, 3, x_23); +x_25 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__16; +lean_inc(x_24); +lean_inc(x_18); +lean_inc(x_10); +x_26 = l_Lean_Syntax_node2(x_10, x_25, x_18, x_24); +x_27 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__40; +lean_inc(x_10); +x_28 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_28, 0, x_10); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7; +lean_inc(x_10); +x_30 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_30, 0, x_10); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8; +lean_inc(x_10); +x_32 = l_Lean_Syntax_node1(x_10, x_31, x_30); +x_33 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9; +lean_inc(x_10); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_10); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10; +lean_inc(x_10); +x_36 = l_Lean_Syntax_node1(x_10, x_35, x_34); +x_37 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__7; +lean_inc(x_32); +lean_inc(x_28); +lean_inc(x_10); +x_38 = l_Lean_Syntax_node5(x_10, x_37, x_26, x_28, x_32, x_28, x_36); +x_39 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__14; +lean_inc(x_10); +x_40 = l_Lean_Syntax_node1(x_10, x_39, x_38); +x_41 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__12; +lean_inc(x_10); +x_42 = l_Lean_Syntax_node1(x_10, x_41, x_40); +x_43 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__9; +lean_inc(x_16); +lean_inc(x_10); +x_44 = l_Lean_Syntax_node2(x_10, x_43, x_16, x_42); +x_45 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__30; +lean_inc(x_11); +lean_inc(x_12); +x_46 = l_Lean_addMacroScope(x_12, x_45, x_11); +x_47 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__27; +x_48 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__32; +lean_inc(x_10); +x_49 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_49, 0, x_10); +lean_ctor_set(x_49, 1, x_47); +lean_ctor_set(x_49, 2, x_46); +lean_ctor_set(x_49, 3, x_48); +x_50 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__35; +lean_inc(x_10); +x_51 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_51, 0, x_10); +lean_ctor_set(x_51, 1, x_50); +x_52 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13; +lean_inc(x_10); +x_53 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_53, 0, x_10); +lean_ctor_set(x_53, 1, x_52); +x_54 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16; +x_55 = l_Lean_addMacroScope(x_12, x_54, x_11); +x_56 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15; +lean_inc(x_10); +x_57 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_57, 0, x_10); +lean_ctor_set(x_57, 1, x_56); +lean_ctor_set(x_57, 2, x_55); +lean_ctor_set(x_57, 3, x_21); +x_58 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12; +lean_inc(x_57); +lean_inc(x_10); +x_59 = l_Lean_Syntax_node2(x_10, x_58, x_53, x_57); +lean_inc(x_10); +x_60 = l_Lean_Syntax_node1(x_10, x_37, x_59); +x_61 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__25; +lean_inc(x_10); +x_62 = l_Lean_Syntax_node2(x_10, x_61, x_24, x_60); +x_63 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__39; +lean_inc(x_10); +x_64 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_64, 0, x_10); +lean_ctor_set(x_64, 1, x_63); +x_65 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__34; +lean_inc(x_10); +x_66 = l_Lean_Syntax_node3(x_10, x_65, x_51, x_62, x_64); +lean_inc(x_10); +x_67 = l_Lean_Syntax_node1(x_10, x_37, x_66); +lean_inc(x_10); +x_68 = l_Lean_Syntax_node2(x_10, x_61, x_49, x_67); +lean_inc(x_10); +x_69 = l_Lean_Syntax_node2(x_10, x_25, x_18, x_68); +x_70 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__44; +lean_inc(x_10); +x_71 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_71, 0, x_10); +lean_ctor_set(x_71, 1, x_37); +lean_ctor_set(x_71, 2, x_70); +x_72 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17; +lean_inc(x_10); +x_73 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_73, 0, x_10); +lean_ctor_set(x_73, 1, x_72); +x_74 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22; +lean_inc(x_10); +x_75 = l_Lean_Syntax_node1(x_10, x_74, x_57); +x_76 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20; +lean_inc(x_71); +lean_inc(x_10); +x_77 = l_Lean_Syntax_node2(x_10, x_76, x_75, x_71); +lean_inc(x_10); +x_78 = l_Lean_Syntax_node1(x_10, x_37, x_77); +x_79 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23; +lean_inc(x_10); +x_80 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_80, 0, x_10); +lean_ctor_set(x_80, 1, x_79); +lean_inc(x_10); +x_81 = l_Lean_Syntax_node1(x_10, x_37, x_32); +lean_inc(x_10); +x_82 = l_Lean_Syntax_node1(x_10, x_39, x_81); +lean_inc(x_10); +x_83 = l_Lean_Syntax_node1(x_10, x_41, x_82); +x_84 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18; +lean_inc(x_10); +x_85 = l_Lean_Syntax_node4(x_10, x_84, x_73, x_78, x_80, x_83); +x_86 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__43; +lean_inc(x_10); +x_87 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_87, 0, x_10); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__42; +lean_inc_n(x_71, 5); +lean_inc(x_10); +x_89 = l_Lean_Syntax_node6(x_10, x_88, x_87, x_71, x_71, x_71, x_71, x_71); +lean_inc(x_71); +lean_inc(x_10); +x_90 = l_Lean_Syntax_node5(x_10, x_37, x_69, x_71, x_85, x_71, x_89); +lean_inc(x_10); +x_91 = l_Lean_Syntax_node1(x_10, x_39, x_90); +lean_inc(x_10); +x_92 = l_Lean_Syntax_node1(x_10, x_41, x_91); +lean_inc(x_10); +x_93 = l_Lean_Syntax_node2(x_10, x_43, x_16, x_92); +lean_inc(x_10); +x_94 = l_Lean_Syntax_node2(x_10, x_37, x_44, x_93); +x_95 = l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__5; +x_96 = l_Lean_Syntax_node2(x_10, x_95, x_14, x_94); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_3); +return x_97; +} +} +} +LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__2; +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; 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; +x_8 = lean_ctor_get(x_2, 5); +lean_inc(x_8); +lean_dec(x_2); +x_9 = 0; +x_10 = l_Lean_SourceInfo_fromRef(x_8, x_9); +x_11 = l_Array_tacticArray__mem__dec___closed__3; +lean_inc(x_10); +x_12 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_11); +x_13 = l_Array_tacticArray__mem__dec___closed__2; +x_14 = l_Lean_Syntax_node1(x_10, x_13, x_12); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_3); +return x_15; +} +} +} lean_object* initialize_Init_Data_Array_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Nat_Linear(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_BasicAux(uint8_t builtin, lean_object*); @@ -964,6 +1519,64 @@ l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__1); l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__2 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__2(); lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__tacticDecreasing__trivial__1___closed__2); +l_Array_tacticArray__mem__dec___closed__1 = _init_l_Array_tacticArray__mem__dec___closed__1(); +lean_mark_persistent(l_Array_tacticArray__mem__dec___closed__1); +l_Array_tacticArray__mem__dec___closed__2 = _init_l_Array_tacticArray__mem__dec___closed__2(); +lean_mark_persistent(l_Array_tacticArray__mem__dec___closed__2); +l_Array_tacticArray__mem__dec___closed__3 = _init_l_Array_tacticArray__mem__dec___closed__3(); +lean_mark_persistent(l_Array_tacticArray__mem__dec___closed__3); +l_Array_tacticArray__mem__dec___closed__4 = _init_l_Array_tacticArray__mem__dec___closed__4(); +lean_mark_persistent(l_Array_tacticArray__mem__dec___closed__4); +l_Array_tacticArray__mem__dec___closed__5 = _init_l_Array_tacticArray__mem__dec___closed__5(); +lean_mark_persistent(l_Array_tacticArray__mem__dec___closed__5); +l_Array_tacticArray__mem__dec = _init_l_Array_tacticArray__mem__dec(); +lean_mark_persistent(l_Array_tacticArray__mem__dec); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__1); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__2); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__3); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__4); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__5); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__6); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__7); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__8); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__9); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__10); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__11); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__12); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__13); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__14); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__15); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__16); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__17); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__18); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__19); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__20); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__22); +l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23 = _init_l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23(); +lean_mark_persistent(l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__23); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Data/List/Basic.c b/stage0/stdlib/Init/Data/List/Basic.c index d3789647c6a4..86159a8cb405 100644 --- a/stage0/stdlib/Init/Data/List/Basic.c +++ b/stage0/stdlib/Init/Data/List/Basic.c @@ -44,7 +44,6 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_concat_match__ LEAN_EXPORT lean_object* l_List_eraseDups_loop(lean_object*); LEAN_EXPORT lean_object* l_List_unzip___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_concat_match__1_splitter(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1(lean_object*); LEAN_EXPORT lean_object* l_List_reverseAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_zipWith___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_elem(lean_object*); @@ -77,9 +76,8 @@ LEAN_EXPORT lean_object* l_List_and___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdx___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instLTList(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_isEqv___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_instDecidableMemListInstMembershipList___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_instDecidableMemListInstMembershipList___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_beq___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_intersperse_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -165,10 +163,9 @@ LEAN_EXPORT lean_object* l_List_elem___rarg___boxed(lean_object*, lean_object*, LEAN_EXPORT lean_object* l_List_lookup(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instGetElemListNatLtInstLTNatLength(lean_object*); LEAN_EXPORT lean_object* l_List_groupBy_loop(lean_object*); -LEAN_EXPORT lean_object* l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filter(lean_object*); LEAN_EXPORT lean_object* l_List_isSuffixOf(lean_object*); -LEAN_EXPORT uint8_t l_List_instDecidableMemListInstMembershipList___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_List_instDecidableMemListInstMembershipList___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instLEList___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_length_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_List_removeAll___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1870,87 +1867,29 @@ x_2 = lean_box(0); return x_2; } } -LEAN_EXPORT uint8_t l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_List_instDecidableMemListInstMembershipList___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -if (lean_obj_tag(x_3) == 0) -{ -uint8_t x_4; -lean_dec(x_2); -lean_dec(x_1); -x_4 = 0; -return x_4; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_3, 1); -lean_inc(x_6); -lean_dec(x_3); -lean_inc(x_1); -lean_inc(x_2); -x_7 = lean_apply_2(x_1, x_2, x_5); -x_8 = lean_unbox(x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -x_3 = x_6; -goto _start; -} -else -{ -uint8_t x_10; -lean_dec(x_6); -lean_dec(x_2); -lean_dec(x_1); -x_10 = 1; -return x_10; -} -} -} -} -LEAN_EXPORT lean_object* l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg___boxed), 3, 0); -return x_2; -} -} -LEAN_EXPORT uint8_t l_List_instDecidableMemListInstMembershipList___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg(x_1, x_2, x_3); -return x_4; +uint8_t x_5; +x_5 = l_List_elem___rarg(x_1, x_3, x_4); +return x_5; } } LEAN_EXPORT lean_object* l_List_instDecidableMemListInstMembershipList(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_instDecidableMemListInstMembershipList___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_List_instDecidableMemListInstMembershipList___rarg___boxed), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_instDecidableMemListInstMembershipList___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -uint8_t x_4; lean_object* x_5; -x_4 = l_List_elem___at_List_instDecidableMemListInstMembershipList___spec__1___rarg(x_1, x_2, x_3); -x_5 = lean_box(x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_List_instDecidableMemListInstMembershipList___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = l_List_instDecidableMemListInstMembershipList___rarg(x_1, x_2, x_3); -x_5 = lean_box(x_4); -return x_5; +uint8_t x_5; lean_object* x_6; +x_5 = l_List_instDecidableMemListInstMembershipList___rarg(x_1, x_2, x_3, x_4); +x_6 = lean_box(x_5); +return x_6; } } LEAN_EXPORT lean_object* l_List_eraseDups_loop___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { diff --git a/stage0/stdlib/Init/Meta.c b/stage0/stdlib/Init/Meta.c index 7eeff41718e0..f3ba4588d3c0 100644 --- a/stage0/stdlib/Init/Meta.c +++ b/stage0/stdlib/Init/Meta.c @@ -27,8 +27,11 @@ lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Name_instDecidableEqName(lean_object*, lean_object*); static lean_object* l_Lean_instQuoteSubstringMkStr1___closed__2; static lean_object* l_Lean_mkGroupNode___closed__2; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8; LEAN_EXPORT lean_object* l_Lean_instQuote(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__outOfBounds___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21180_(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1; static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__7; LEAN_EXPORT lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailArraySyntaxTSepArray___boxed(lean_object*); @@ -81,6 +84,7 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_isNameLit_x3f___boxed(lean_object*); static lean_object* l_Lean_instQuoteBoolMkStr1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_dsimpKind; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeExp___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__5; LEAN_EXPORT lean_object* l_Lean_Syntax_instReprTSyntax(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__12; @@ -126,7 +130,6 @@ extern lean_object* l_Lean_maxRecDepthErrorMessage; static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____closed__22; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; static lean_object* l_Lean_Syntax_instCoeIdentTSyntaxConsSyntaxNodeKindMkStr4Nil___closed__3; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18173_(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_toString___boxed(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -141,7 +144,6 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeOutTSyntaxArrayArraySyntax(lean_ob static lean_object* l_Lean_Parser_Tactic_simpArith___closed__4; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decode(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_Tactic_location; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5; static lean_object* l_Lean_evalPrec___closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602____closed__3; @@ -152,6 +154,7 @@ static lean_object* l_Lean_Syntax_mkNumLit___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__21; LEAN_EXPORT lean_object* l_repr___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__2___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__80; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18265_(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_getString(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrec(lean_object*); @@ -183,7 +186,6 @@ LEAN_EXPORT lean_object* l_Lean_Option_hasQuote(lean_object*); LEAN_EXPORT lean_object* l_Lean_NameGenerator_curr(lean_object*); LEAN_EXPORT lean_object* l_Lean_monadNameGeneratorLift___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_version_major___closed__1; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7; static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602____closed__21; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeStrLitTerm(lean_object*); @@ -197,7 +199,6 @@ static lean_object* l_Lean_TSyntax_expandInterpolatedStr___closed__2; static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602_(uint8_t, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__5; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_TSyntax_expandInterpolatedStrChunks___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkIdentFrom___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeArraySyntaxSepArray(lean_object*); @@ -214,6 +215,7 @@ uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__32; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__110; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__73; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__79; LEAN_EXPORT lean_object* l_List_repr___at___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____spec__4___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkCIdentFrom___boxed(lean_object*, lean_object*, lean_object*); @@ -221,13 +223,14 @@ static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__2; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst___at_Lean_Syntax_setHeadInfoAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__10; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__58; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_isScientificLit_x3f___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__12; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeIdentTerm(lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); static lean_object* l_Lean_version_specialDesc___closed__1; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__19; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__69; static lean_object* l_Lean_Syntax_instReprTSyntax___closed__1; @@ -245,7 +248,6 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeOutTSepArrayTSyntaxArray(lean_obje LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed__const__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__106; static lean_object* l_Lean_termEval__prio_____closed__7; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20025_(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterSepElemsM(lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); @@ -255,7 +257,6 @@ static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__5; LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionSepArray(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__22; uint8_t l_String_contains(lean_object*, uint32_t); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_isNatLitAux___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__4; @@ -266,7 +267,6 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpAllArith; LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_getElems___rarg___boxed(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4; LEAN_EXPORT lean_object* l_Array_filterSepElems___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__87; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__5; @@ -311,9 +311,9 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__61; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__subPrec__1___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3; LEAN_EXPORT uint32_t l_Lean_idBeginEscape; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__25; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKind___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isGreek___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__6; @@ -341,6 +341,7 @@ static lean_object* l_Lean_termEval__prec_____closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; LEAN_EXPORT uint8_t l_Lean_Syntax_isAtom(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__47; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235_(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Rewrite_Config_offsetCnstrs___default; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeOutTSyntaxArrayArraySyntax___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__3; @@ -384,6 +385,7 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_isInterpolatedStrLit_x3f(lean_object*); static lean_object* l_Lean_versionStringCore___closed__2; LEAN_EXPORT lean_object* l_Lean_Syntax_splitNameLit(lean_object*); static lean_object* l_Lean_TSyntax_expandInterpolatedStr___closed__1; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330_(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_reprTSyntax____x40_Init_Meta___hyg_2618____rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__33; @@ -420,7 +422,6 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArrayTSepArray___rarg___box static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__45; LEAN_EXPORT lean_object* l_Lean_instQuoteBoolMkStr1(uint8_t); LEAN_EXPORT lean_object* l_Lean_Syntax_isIdOrAtom_x3f(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__27; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__5; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__11; @@ -479,7 +480,6 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_getOptionalIdent_x3f___boxed(lean_object* static lean_object* l_Lean_termEval__prec_____closed__3; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__6; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867_(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Syntax_getSepArgs___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__17; @@ -500,6 +500,7 @@ static lean_object* l_Lean_Syntax_isCharLit_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Syntax_isIdOrAtom_x3f___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__8; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeHexLitAux(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__87; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__92; static lean_object* l_Lean_TSyntax_expandInterpolatedStrChunks___closed__1; @@ -542,11 +543,13 @@ static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprTSyntax____x40_Init static lean_object* l_Lean_Syntax_isCharLit_x3f___closed__1; static lean_object* l_Lean_termEval__prio_____closed__9; static lean_object* l_Lean_TSyntax_expandInterpolatedStr___lambda__1___closed__2; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; extern lean_object* l_Lean_Parser_Tactic_simpLemma; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeAfterExp(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkCIdentFromRef___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__4(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__58; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__2; LEAN_EXPORT lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); @@ -564,7 +567,6 @@ static lean_object* l_Lean_Syntax_getHead_x3f___closed__3; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeAfterDot(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_beq_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1; static lean_object* l_Lean_Name_escapePart___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__81; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeDecimalLitAux(lean_object*, lean_object*, lean_object*); @@ -572,18 +574,17 @@ static lean_object* l_Lean_termEval__prec_____closed__6; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__56; static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__9; LEAN_EXPORT lean_object* l_List_foldl___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7; LEAN_EXPORT lean_object* l_Lean_quoteNameMk(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkGroupNode(lean_object*); LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Lean_Syntax_structEq___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__88; LEAN_EXPORT lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeDecimalLitAux___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602____closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_TSyntax_expandInterpolatedStrChunks___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__131; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8; static lean_object* l_Lean_Syntax_instBEqPreresolved___closed__1; static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____closed__17; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getSepElems___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); @@ -599,7 +600,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__32; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__9; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrLit___boxed(lean_object*); @@ -622,6 +622,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__4; static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____closed__8; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__4; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__9; static lean_object* l_Lean_termEval__prio_____closed__1; @@ -652,7 +653,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrLit_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Syntax_getHead_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapSepElemsM___at_Array_mapSepElems___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Syntax_instCoeTSyntaxArray___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Substring_toName(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____boxed(lean_object*, lean_object*); @@ -662,6 +662,7 @@ static lean_object* l_Lean_mkOptionalNode___closed__1; static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__12; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___at_Lean_Syntax_setTailInfoAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__18; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__5; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_beq_match__1_splitter(lean_object*); @@ -701,6 +702,7 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrio(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__57; LEAN_EXPORT lean_object* l_Lean_Syntax_getHead_x3f(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__20; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__8; LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push___boxed(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); @@ -741,7 +743,6 @@ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__51; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__78; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__28; static lean_object* l_Lean_mkSepArray___closed__2; @@ -792,7 +793,6 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_getHygieneInfo(lean_object*); lean_object* l_Lean_MacroScopesView_review(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed__const__1; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6; static lean_object* l_Lean_Syntax_instCoeOutSepArrayArraySyntax___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_isNone___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef(lean_object*); @@ -809,6 +809,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_mkSepArray___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__111; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__16; LEAN_EXPORT lean_object* l_Lean_version_major; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__8; @@ -818,6 +819,7 @@ static lean_object* l_Lean_Syntax_mkScientificLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Syntax_getSubstring_x3f(lean_object*, uint8_t, uint8_t); static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__10; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeIdentTerm___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6; static lean_object* l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__4; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__3; static lean_object* l_Lean_mkHole___closed__2; @@ -842,6 +844,7 @@ static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__10; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_reprTSyntax____x40_Init_Meta___hyg_2618____rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; lean_object* l_Lean_SourceInfo_getPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* lean_name_append_index_after(lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602____closed__7; @@ -879,6 +882,7 @@ LEAN_EXPORT uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__6; static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_12602____closed__13; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__137; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2; static lean_object* l_Lean_instQuoteSubstringMkStr1___closed__1; static lean_object* l_Lean_Name_reprPrec___closed__6; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__136; @@ -938,6 +942,7 @@ LEAN_EXPORT uint8_t l_Lean_Syntax_hasArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_getNat(lean_object*); static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__15; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20209_(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__4; static lean_object* l_List_foldr___at_Substring_toName___spec__1___closed__3; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrLit(lean_object*); @@ -967,6 +972,7 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_Syntax_find_x3f(lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Syntax_reprTSyntax____x40_Init_Meta___hyg_2618____rarg___closed__12; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__119; lean_object* l_id___rarg___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__15; @@ -989,6 +995,7 @@ static lean_object* l_Lean_toolchain___closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_getElems(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteArray___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; lean_object* l_Lean_Syntax_node7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__17; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__38; @@ -1009,12 +1016,12 @@ lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__8; static lean_object* l_Lean_versionString___closed__11; LEAN_EXPORT lean_object* l_Lean_Syntax_findAux(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1; LEAN_EXPORT lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); uint8_t l_String_isPrefixOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Syntax_instCoeTSyntaxArray___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_instToStringName(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__21; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__77; LEAN_EXPORT lean_object* l_Lean_Syntax_isCharLit_x3f(lean_object*); @@ -1047,7 +1054,6 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailArraySyntaxTSyntaxArra static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__118; LEAN_EXPORT lean_object* l_Lean_Name_eraseSuffix_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__44; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__1; LEAN_EXPORT uint8_t l_Lean_isIdEndEscape(uint32_t); @@ -1066,6 +1072,7 @@ static lean_object* l_Lean_mkSepArray___closed__1; static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__7; static lean_object* l_Lean_mkCIdentFrom___closed__2; lean_object* l_Array_mkArray1___rarg(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3; static lean_object* l_Lean_Syntax_mkApp___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__59; lean_object* lean_nat_mul(lean_object*, lean_object*); @@ -1080,6 +1087,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpArith; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Syntax_findAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__6; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeScientificLitTerm___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_termEval__prec_____closed__4; static lean_object* l_Lean_Syntax_mkStrLit___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__82; @@ -1115,7 +1123,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_instQuote___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_instQuoteBoolMkStr1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146_(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instQuoteNameMkStr1___closed__2; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__4; static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; @@ -1129,7 +1136,9 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_beq_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4; LEAN_EXPORT lean_object* l_Lean_instQuoteBoolMkStr1___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrio__1___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__117; LEAN_EXPORT lean_object* l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1(lean_object*, lean_object*); @@ -1167,6 +1176,7 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteList(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__6; lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_repr___at___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_version_getSpecialDesc___boxed(lean_object*); static lean_object* l_Lean_mkOptionalNode___closed__3; @@ -1185,7 +1195,6 @@ extern lean_object* l_Lean_instInhabitedSyntax; static lean_object* l_Lean_versionStringCore___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__115; lean_object* lean_version_get_minor(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__22; static lean_object* l_Lean_Parser_Tactic_declareSimpLikeTactic___closed__17; LEAN_EXPORT lean_object* l_repr___at___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2353____spec__5(lean_object*); @@ -1223,7 +1232,6 @@ lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__26; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeNatLitVal_x3f___boxed(lean_object*); static lean_object* l_Lean_termEval__prec_____closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__72; LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__termEval__prec____1(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_pred(lean_object*); @@ -1261,18 +1269,18 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux___at_Array_mapSepElems___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instQuoteArrayMkStr1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20904_(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_termEval__prio_____closed__2; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__subPrec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_instQuoteStringStrLitKind___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__49; LEAN_EXPORT lean_object* l_Lean_TSyntax_getString___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_toString_maybePseudoSyntax___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_evalPrio___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__14; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___closed__30; LEAN_EXPORT lean_object* l_Lean_Name_toStringWithSep(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_quoteArray_go___rarg___closed__1; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__2; LEAN_EXPORT lean_object* l_Lean_HygieneInfo_mkIdent(lean_object*, lean_object*, uint8_t); @@ -1298,7 +1306,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpAutoUnfold; static lean_object* l_Lean_termEval__prio_____closed__4; static lean_object* l_Lean_Option_hasQuote___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_mkHole___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__135; LEAN_EXPORT lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); @@ -25395,6 +25402,75 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("decide", 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Decidable", 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -25409,7 +25485,7 @@ lean_inc(x_7); x_9 = l_Lean_Syntax_isOfKind(x_7, x_8); if (x_9 == 0) { -lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_dec(x_7); x_10 = lean_ctor_get(x_2, 5); lean_inc(x_10); @@ -25525,6 +25601,8 @@ lean_inc(x_43); lean_inc(x_12); x_57 = l_Lean_Syntax_node2(x_12, x_56, x_55, x_43); x_58 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; +lean_inc(x_13); +lean_inc(x_14); x_59 = l_Lean_addMacroScope(x_14, x_58, x_13); x_60 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; x_61 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; @@ -25535,218 +25613,264 @@ lean_ctor_set(x_62, 1, x_60); lean_ctor_set(x_62, 2, x_59); lean_ctor_set(x_62, 3, x_61); x_63 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_62); lean_inc(x_20); lean_inc(x_12); x_64 = l_Lean_Syntax_node3(x_12, x_63, x_57, x_20, x_62); +x_65 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; lean_inc(x_12); -x_65 = l_Lean_Syntax_node1(x_12, x_35, x_64); -x_66 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +x_66 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_66, 0, x_12); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_68 = l_Lean_addMacroScope(x_14, x_67, x_13); +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_70 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_12); +x_71 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_71, 0, x_12); +lean_ctor_set(x_71, 1, x_69); +lean_ctor_set(x_71, 2, x_68); +lean_ctor_set(x_71, 3, x_70); lean_inc(x_43); lean_inc(x_12); -x_67 = l_Lean_Syntax_node1(x_12, x_66, x_43); -x_68 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +x_72 = l_Lean_Syntax_node2(x_12, x_56, x_71, x_43); +lean_inc(x_20); lean_inc(x_12); -x_69 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_69, 0, x_12); -lean_ctor_set(x_69, 1, x_68); -x_70 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_69); +x_73 = l_Lean_Syntax_node3(x_12, x_63, x_72, x_20, x_62); +lean_inc(x_12); +x_74 = l_Lean_Syntax_node3(x_12, x_35, x_64, x_66, x_73); +x_75 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; lean_inc(x_43); -lean_inc(x_67); +lean_inc(x_12); +x_76 = l_Lean_Syntax_node1(x_12, x_75, x_43); +x_77 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_12); +x_78 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_78, 0, x_12); +lean_ctor_set(x_78, 1, x_77); +x_79 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_78); +lean_inc(x_43); +lean_inc(x_76); lean_inc(x_47); lean_inc(x_12); -x_71 = l_Lean_Syntax_node6(x_12, x_70, x_47, x_51, x_65, x_67, x_43, x_69); -x_72 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +x_80 = l_Lean_Syntax_node6(x_12, x_79, x_47, x_51, x_74, x_76, x_43, x_78); +x_81 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; lean_inc(x_43); lean_inc(x_12); -x_73 = l_Lean_Syntax_node4(x_12, x_72, x_41, x_43, x_45, x_71); -x_74 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +x_82 = l_Lean_Syntax_node4(x_12, x_81, x_41, x_43, x_45, x_80); +x_83 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; lean_inc(x_12); -x_75 = l_Lean_Syntax_node2(x_12, x_74, x_22, x_73); -x_76 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; -lean_inc(x_69); +x_84 = l_Lean_Syntax_node2(x_12, x_83, x_22, x_82); +x_85 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; +lean_inc(x_78); lean_inc(x_47); lean_inc(x_12); -x_77 = l_Lean_Syntax_node2(x_12, x_76, x_47, x_69); +x_86 = l_Lean_Syntax_node2(x_12, x_85, x_47, x_78); lean_inc_n(x_43, 2); lean_inc(x_12); -x_78 = l_Lean_Syntax_node6(x_12, x_70, x_47, x_43, x_43, x_67, x_43, x_69); -x_79 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; +x_87 = l_Lean_Syntax_node6(x_12, x_79, x_47, x_43, x_43, x_76, x_43, x_78); +x_88 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; lean_inc(x_12); -x_80 = l_Lean_Syntax_node2(x_12, x_79, x_77, x_78); +x_89 = l_Lean_Syntax_node2(x_12, x_88, x_86, x_87); lean_inc(x_12); -x_81 = l_Lean_Syntax_node1(x_12, x_35, x_80); -x_82 = l_Lean_Syntax_mkApp___closed__2; +x_90 = l_Lean_Syntax_node1(x_12, x_35, x_89); +x_91 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); -x_83 = l_Lean_Syntax_node2(x_12, x_82, x_75, x_81); -x_84 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_83, x_38); -x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_84, x_2, x_3); +x_92 = l_Lean_Syntax_node2(x_12, x_91, x_84, x_90); +x_93 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_92, x_38); +x_94 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_93, x_2, x_3); lean_dec(x_2); -return x_85; +return x_94; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t 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; -x_86 = lean_unsigned_to_nat(3u); -x_87 = l_Lean_Syntax_getArg(x_7, x_86); +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; 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; +x_95 = lean_unsigned_to_nat(3u); +x_96 = l_Lean_Syntax_getArg(x_7, x_95); lean_dec(x_7); -x_88 = lean_ctor_get(x_2, 5); -lean_inc(x_88); -x_89 = 0; -x_90 = l_Lean_SourceInfo_fromRef(x_88, x_89); -x_91 = lean_ctor_get(x_2, 2); -lean_inc(x_91); -x_92 = lean_ctor_get(x_2, 1); -lean_inc(x_92); -x_93 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; -lean_inc(x_90); -x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_90); -lean_ctor_set(x_94, 1, x_93); -x_95 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; -lean_inc(x_90); -x_96 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_96, 0, x_90); -lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; -lean_inc(x_90); -x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_90); -lean_ctor_set(x_98, 1, x_97); -x_99 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; -lean_inc(x_90); -x_100 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_100, 0, x_90); -lean_ctor_set(x_100, 1, x_99); -x_101 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; -lean_inc(x_91); -lean_inc(x_92); -x_102 = l_Lean_addMacroScope(x_92, x_101, x_91); -x_103 = lean_box(0); -x_104 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; -lean_inc(x_90); -x_105 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_105, 0, x_90); +x_97 = lean_ctor_get(x_2, 5); +lean_inc(x_97); +x_98 = 0; +x_99 = l_Lean_SourceInfo_fromRef(x_97, x_98); +x_100 = lean_ctor_get(x_2, 2); +lean_inc(x_100); +x_101 = lean_ctor_get(x_2, 1); +lean_inc(x_101); +x_102 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; +lean_inc(x_99); +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_99); +lean_ctor_set(x_103, 1, x_102); +x_104 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; +lean_inc(x_99); +x_105 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_105, 0, x_99); lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_102); -lean_ctor_set(x_105, 3, x_103); -x_106 = l_Lean_toolchain___closed__1; -lean_inc(x_90); +x_106 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; +lean_inc(x_99); x_107 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_107, 0, x_90); +lean_ctor_set(x_107, 0, x_99); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__6; -lean_inc(x_91); -lean_inc(x_92); -x_109 = l_Lean_addMacroScope(x_92, x_108, x_91); -x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__2; -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__10; -lean_inc(x_90); -x_112 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_112, 0, x_90); -lean_ctor_set(x_112, 1, x_110); -lean_ctor_set(x_112, 2, x_109); -lean_ctor_set(x_112, 3, x_111); -x_113 = l_Lean_mkOptionalNode___closed__2; -lean_inc(x_90); -x_114 = l_Lean_Syntax_node1(x_90, x_113, x_112); -x_115 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; -lean_inc(x_90); +x_108 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; +lean_inc(x_99); +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_99); +lean_ctor_set(x_109, 1, x_108); +x_110 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; +lean_inc(x_100); +lean_inc(x_101); +x_111 = l_Lean_addMacroScope(x_101, x_110, x_100); +x_112 = lean_box(0); +x_113 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; +lean_inc(x_99); +x_114 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_114, 0, x_99); +lean_ctor_set(x_114, 1, x_113); +lean_ctor_set(x_114, 2, x_111); +lean_ctor_set(x_114, 3, x_112); +x_115 = l_Lean_toolchain___closed__1; +lean_inc(x_99); x_116 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_116, 0, x_90); +lean_ctor_set(x_116, 0, x_99); lean_ctor_set(x_116, 1, x_115); -x_117 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; -lean_inc(x_116); -lean_inc(x_105); -lean_inc(x_94); -lean_inc(x_90); -x_118 = l_Lean_Syntax_node5(x_90, x_117, x_94, x_105, x_107, x_114, x_116); -lean_inc(x_90); -x_119 = l_Lean_Syntax_node1(x_90, x_113, x_118); -x_120 = l_Lean_mkSepArray___closed__1; -lean_inc(x_90); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_90); -lean_ctor_set(x_121, 1, x_113); -lean_ctor_set(x_121, 2, x_120); -x_122 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; -lean_inc(x_90); -x_123 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_123, 0, x_90); -lean_ctor_set(x_123, 1, x_122); -x_124 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; -lean_inc(x_90); +x_117 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__6; +lean_inc(x_100); +lean_inc(x_101); +x_118 = l_Lean_addMacroScope(x_101, x_117, x_100); +x_119 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__2; +x_120 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__10; +lean_inc(x_99); +x_121 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_121, 0, x_99); +lean_ctor_set(x_121, 1, x_119); +lean_ctor_set(x_121, 2, x_118); +lean_ctor_set(x_121, 3, x_120); +x_122 = l_Lean_mkOptionalNode___closed__2; +lean_inc(x_99); +x_123 = l_Lean_Syntax_node1(x_99, x_122, x_121); +x_124 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; +lean_inc(x_99); x_125 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_125, 0, x_90); +lean_ctor_set(x_125, 0, x_99); lean_ctor_set(x_125, 1, x_124); -lean_inc(x_90); -x_126 = l_Lean_Syntax_node1(x_90, x_113, x_105); -x_127 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; -lean_inc(x_90); -x_128 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_128, 0, x_90); -lean_ctor_set(x_128, 1, x_127); -lean_inc(x_90); -x_129 = l_Lean_Syntax_node2(x_90, x_113, x_126, x_128); -x_130 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; -lean_inc(x_91); -lean_inc(x_92); -x_131 = l_Lean_addMacroScope(x_92, x_130, x_91); -x_132 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; -lean_inc(x_90); -x_133 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_133, 0, x_90); -lean_ctor_set(x_133, 1, x_132); -lean_ctor_set(x_133, 2, x_131); -lean_ctor_set(x_133, 3, x_103); -x_134 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; -lean_inc(x_121); -lean_inc(x_90); -x_135 = l_Lean_Syntax_node2(x_90, x_134, x_133, x_121); -x_136 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; -x_137 = l_Lean_addMacroScope(x_92, x_136, x_91); -x_138 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; -x_139 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; -lean_inc(x_90); -x_140 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_140, 0, x_90); -lean_ctor_set(x_140, 1, x_138); -lean_ctor_set(x_140, 2, x_137); -lean_ctor_set(x_140, 3, x_139); -x_141 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; -lean_inc(x_98); -lean_inc(x_90); -x_142 = l_Lean_Syntax_node3(x_90, x_141, x_135, x_98, x_140); -lean_inc(x_90); -x_143 = l_Lean_Syntax_node1(x_90, x_113, x_142); -x_144 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; -lean_inc(x_121); -lean_inc(x_90); -x_145 = l_Lean_Syntax_node1(x_90, x_144, x_121); -x_146 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; -lean_inc(x_90); -x_147 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_147, 0, x_90); -lean_ctor_set(x_147, 1, x_146); -x_148 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_121); -lean_inc(x_90); -x_149 = l_Lean_Syntax_node6(x_90, x_148, x_125, x_129, x_143, x_145, x_121, x_147); -x_150 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; -lean_inc(x_90); -x_151 = l_Lean_Syntax_node4(x_90, x_150, x_119, x_121, x_123, x_149); -x_152 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; -lean_inc(x_90); -x_153 = l_Lean_Syntax_node2(x_90, x_152, x_100, x_151); -lean_inc(x_90); -x_154 = l_Lean_Syntax_node1(x_90, x_113, x_87); -x_155 = l_Lean_Syntax_mkApp___closed__2; -lean_inc(x_90); -x_156 = l_Lean_Syntax_node2(x_90, x_155, x_153, x_154); -x_157 = l_Lean_Syntax_node5(x_90, x_8, x_94, x_96, x_98, x_156, x_116); -x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_157, x_2, x_3); +x_126 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; +lean_inc(x_125); +lean_inc(x_114); +lean_inc(x_103); +lean_inc(x_99); +x_127 = l_Lean_Syntax_node5(x_99, x_126, x_103, x_114, x_116, x_123, x_125); +lean_inc(x_99); +x_128 = l_Lean_Syntax_node1(x_99, x_122, x_127); +x_129 = l_Lean_mkSepArray___closed__1; +lean_inc(x_99); +x_130 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_130, 0, x_99); +lean_ctor_set(x_130, 1, x_122); +lean_ctor_set(x_130, 2, x_129); +x_131 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; +lean_inc(x_99); +x_132 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_132, 0, x_99); +lean_ctor_set(x_132, 1, x_131); +x_133 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; +lean_inc(x_99); +x_134 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_134, 0, x_99); +lean_ctor_set(x_134, 1, x_133); +lean_inc(x_99); +x_135 = l_Lean_Syntax_node1(x_99, x_122, x_114); +x_136 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; +lean_inc(x_99); +x_137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_137, 0, x_99); +lean_ctor_set(x_137, 1, x_136); +lean_inc(x_99); +x_138 = l_Lean_Syntax_node2(x_99, x_122, x_135, x_137); +x_139 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; +lean_inc(x_100); +lean_inc(x_101); +x_140 = l_Lean_addMacroScope(x_101, x_139, x_100); +x_141 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; +lean_inc(x_99); +x_142 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_142, 0, x_99); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +lean_ctor_set(x_142, 3, x_112); +x_143 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; +lean_inc(x_130); +lean_inc(x_99); +x_144 = l_Lean_Syntax_node2(x_99, x_143, x_142, x_130); +x_145 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; +lean_inc(x_100); +lean_inc(x_101); +x_146 = l_Lean_addMacroScope(x_101, x_145, x_100); +x_147 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; +x_148 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; +lean_inc(x_99); +x_149 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_149, 0, x_99); +lean_ctor_set(x_149, 1, x_147); +lean_ctor_set(x_149, 2, x_146); +lean_ctor_set(x_149, 3, x_148); +x_150 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_149); +lean_inc(x_107); +lean_inc(x_99); +x_151 = l_Lean_Syntax_node3(x_99, x_150, x_144, x_107, x_149); +x_152 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; +lean_inc(x_99); +x_153 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_153, 0, x_99); +lean_ctor_set(x_153, 1, x_152); +x_154 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_155 = l_Lean_addMacroScope(x_101, x_154, x_100); +x_156 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_157 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_99); +x_158 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_158, 0, x_99); +lean_ctor_set(x_158, 1, x_156); +lean_ctor_set(x_158, 2, x_155); +lean_ctor_set(x_158, 3, x_157); +lean_inc(x_130); +lean_inc(x_99); +x_159 = l_Lean_Syntax_node2(x_99, x_143, x_158, x_130); +lean_inc(x_107); +lean_inc(x_99); +x_160 = l_Lean_Syntax_node3(x_99, x_150, x_159, x_107, x_149); +lean_inc(x_99); +x_161 = l_Lean_Syntax_node3(x_99, x_122, x_151, x_153, x_160); +x_162 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +lean_inc(x_130); +lean_inc(x_99); +x_163 = l_Lean_Syntax_node1(x_99, x_162, x_130); +x_164 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_99); +x_165 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_165, 0, x_99); +lean_ctor_set(x_165, 1, x_164); +x_166 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_130); +lean_inc(x_99); +x_167 = l_Lean_Syntax_node6(x_99, x_166, x_134, x_138, x_161, x_163, x_130, x_165); +x_168 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +lean_inc(x_99); +x_169 = l_Lean_Syntax_node4(x_99, x_168, x_128, x_130, x_132, x_167); +x_170 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +lean_inc(x_99); +x_171 = l_Lean_Syntax_node2(x_99, x_170, x_109, x_169); +lean_inc(x_99); +x_172 = l_Lean_Syntax_node1(x_99, x_122, x_96); +x_173 = l_Lean_Syntax_mkApp___closed__2; +lean_inc(x_99); +x_174 = l_Lean_Syntax_node2(x_99, x_173, x_171, x_172); +x_175 = l_Lean_Syntax_node5(x_99, x_8, x_103, x_105, x_107, x_174, x_125); +x_176 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_175, x_2, x_3); lean_dec(x_2); -return x_158; +return x_176; } } } @@ -25882,7 +26006,7 @@ x_1 = l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__10; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18173_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18265_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -25896,7 +26020,7 @@ lean_inc(x_7); x_9 = l_Lean_Syntax_isOfKind(x_7, x_8); if (x_9 == 0) { -lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_dec(x_7); x_10 = lean_ctor_get(x_2, 5); lean_inc(x_10); @@ -26034,6 +26158,8 @@ x_66 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_66, 0, x_12); lean_ctor_set(x_66, 1, x_65); x_67 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; +lean_inc(x_13); +lean_inc(x_14); x_68 = l_Lean_addMacroScope(x_14, x_67, x_13); x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; lean_inc(x_12); @@ -26044,242 +26170,280 @@ lean_ctor_set(x_70, 2, x_68); lean_ctor_set(x_70, 3, x_25); lean_inc(x_43); lean_inc(x_12); -x_71 = l_Lean_Syntax_node2(x_12, x_56, x_70, x_43); +x_71 = l_Lean_Syntax_node2(x_12, x_56, x_70, x_43); +lean_inc(x_62); +lean_inc(x_20); +lean_inc(x_12); +x_72 = l_Lean_Syntax_node3(x_12, x_63, x_71, x_20, x_62); +x_73 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_74 = l_Lean_addMacroScope(x_14, x_73, x_13); +x_75 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_76 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_12); +x_77 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_77, 0, x_12); +lean_ctor_set(x_77, 1, x_75); +lean_ctor_set(x_77, 2, x_74); +lean_ctor_set(x_77, 3, x_76); +lean_inc(x_43); +lean_inc(x_12); +x_78 = l_Lean_Syntax_node2(x_12, x_56, x_77, x_43); lean_inc(x_20); lean_inc(x_12); -x_72 = l_Lean_Syntax_node3(x_12, x_63, x_71, x_20, x_62); +x_79 = l_Lean_Syntax_node3(x_12, x_63, x_78, x_20, x_62); +lean_inc(x_66); lean_inc(x_12); -x_73 = l_Lean_Syntax_node3(x_12, x_35, x_64, x_66, x_72); -x_74 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +x_80 = l_Lean_Syntax_node5(x_12, x_35, x_64, x_66, x_72, x_66, x_79); +x_81 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; lean_inc(x_43); lean_inc(x_12); -x_75 = l_Lean_Syntax_node1(x_12, x_74, x_43); -x_76 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +x_82 = l_Lean_Syntax_node1(x_12, x_81, x_43); +x_83 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; lean_inc(x_12); -x_77 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_77, 0, x_12); -lean_ctor_set(x_77, 1, x_76); -x_78 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_77); +x_84 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_84, 0, x_12); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_84); lean_inc(x_43); -lean_inc(x_75); +lean_inc(x_82); lean_inc(x_47); lean_inc(x_12); -x_79 = l_Lean_Syntax_node6(x_12, x_78, x_47, x_51, x_73, x_75, x_43, x_77); -x_80 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +x_86 = l_Lean_Syntax_node6(x_12, x_85, x_47, x_51, x_80, x_82, x_43, x_84); +x_87 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; lean_inc(x_43); lean_inc(x_12); -x_81 = l_Lean_Syntax_node4(x_12, x_80, x_41, x_43, x_45, x_79); -x_82 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +x_88 = l_Lean_Syntax_node4(x_12, x_87, x_41, x_43, x_45, x_86); +x_89 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; lean_inc(x_12); -x_83 = l_Lean_Syntax_node2(x_12, x_82, x_22, x_81); -x_84 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; -lean_inc(x_77); +x_90 = l_Lean_Syntax_node2(x_12, x_89, x_22, x_88); +x_91 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; +lean_inc(x_84); lean_inc(x_47); lean_inc(x_12); -x_85 = l_Lean_Syntax_node2(x_12, x_84, x_47, x_77); +x_92 = l_Lean_Syntax_node2(x_12, x_91, x_47, x_84); lean_inc_n(x_43, 2); lean_inc(x_12); -x_86 = l_Lean_Syntax_node6(x_12, x_78, x_47, x_43, x_43, x_75, x_43, x_77); -x_87 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; +x_93 = l_Lean_Syntax_node6(x_12, x_85, x_47, x_43, x_43, x_82, x_43, x_84); +x_94 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; lean_inc(x_12); -x_88 = l_Lean_Syntax_node2(x_12, x_87, x_85, x_86); +x_95 = l_Lean_Syntax_node2(x_12, x_94, x_92, x_93); lean_inc(x_12); -x_89 = l_Lean_Syntax_node1(x_12, x_35, x_88); -x_90 = l_Lean_Syntax_mkApp___closed__2; +x_96 = l_Lean_Syntax_node1(x_12, x_35, x_95); +x_97 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); -x_91 = l_Lean_Syntax_node2(x_12, x_90, x_83, x_89); -x_92 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_91, x_38); -x_93 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_92, x_2, x_3); +x_98 = l_Lean_Syntax_node2(x_12, x_97, x_90, x_96); +x_99 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_98, x_38); +x_100 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_99, x_2, x_3); lean_dec(x_2); -return x_93; +return x_100; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; 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; -x_94 = lean_unsigned_to_nat(3u); -x_95 = l_Lean_Syntax_getArg(x_7, x_94); +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; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; +x_101 = lean_unsigned_to_nat(3u); +x_102 = l_Lean_Syntax_getArg(x_7, x_101); lean_dec(x_7); -x_96 = lean_ctor_get(x_2, 5); -lean_inc(x_96); -x_97 = 0; -x_98 = l_Lean_SourceInfo_fromRef(x_96, x_97); -x_99 = lean_ctor_get(x_2, 2); -lean_inc(x_99); -x_100 = lean_ctor_get(x_2, 1); -lean_inc(x_100); -x_101 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; -lean_inc(x_98); -x_102 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_102, 0, x_98); -lean_ctor_set(x_102, 1, x_101); -x_103 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; -lean_inc(x_98); -x_104 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_104, 0, x_98); -lean_ctor_set(x_104, 1, x_103); -x_105 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; -lean_inc(x_98); -x_106 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_106, 0, x_98); -lean_ctor_set(x_106, 1, x_105); -x_107 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; -lean_inc(x_98); -x_108 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_108, 0, x_98); -lean_ctor_set(x_108, 1, x_107); -x_109 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; -lean_inc(x_99); -lean_inc(x_100); -x_110 = l_Lean_addMacroScope(x_100, x_109, x_99); -x_111 = lean_box(0); -x_112 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; -lean_inc(x_98); -x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_98); +x_103 = lean_ctor_get(x_2, 5); +lean_inc(x_103); +x_104 = 0; +x_105 = l_Lean_SourceInfo_fromRef(x_103, x_104); +x_106 = lean_ctor_get(x_2, 2); +lean_inc(x_106); +x_107 = lean_ctor_get(x_2, 1); +lean_inc(x_107); +x_108 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; +lean_inc(x_105); +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_105); +lean_ctor_set(x_109, 1, x_108); +x_110 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; +lean_inc(x_105); +x_111 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_111, 0, x_105); +lean_ctor_set(x_111, 1, x_110); +x_112 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; +lean_inc(x_105); +x_113 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_113, 0, x_105); lean_ctor_set(x_113, 1, x_112); -lean_ctor_set(x_113, 2, x_110); -lean_ctor_set(x_113, 3, x_111); -x_114 = l_Lean_toolchain___closed__1; -lean_inc(x_98); +x_114 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; +lean_inc(x_105); x_115 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_115, 0, x_98); +lean_ctor_set(x_115, 0, x_105); lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__6; -lean_inc(x_99); -lean_inc(x_100); -x_117 = l_Lean_addMacroScope(x_100, x_116, x_99); -x_118 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__2; -x_119 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__10; -lean_inc(x_98); +x_116 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; +lean_inc(x_106); +lean_inc(x_107); +x_117 = l_Lean_addMacroScope(x_107, x_116, x_106); +x_118 = lean_box(0); +x_119 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; +lean_inc(x_105); x_120 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_120, 0, x_98); -lean_ctor_set(x_120, 1, x_118); +lean_ctor_set(x_120, 0, x_105); +lean_ctor_set(x_120, 1, x_119); lean_ctor_set(x_120, 2, x_117); -lean_ctor_set(x_120, 3, x_119); -x_121 = l_Lean_mkOptionalNode___closed__2; -lean_inc(x_98); -x_122 = l_Lean_Syntax_node1(x_98, x_121, x_120); -x_123 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; -lean_inc(x_98); -x_124 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_124, 0, x_98); -lean_ctor_set(x_124, 1, x_123); -x_125 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; -lean_inc(x_124); -lean_inc(x_113); -lean_inc(x_102); -lean_inc(x_98); -x_126 = l_Lean_Syntax_node5(x_98, x_125, x_102, x_113, x_115, x_122, x_124); -lean_inc(x_98); -x_127 = l_Lean_Syntax_node1(x_98, x_121, x_126); -x_128 = l_Lean_mkSepArray___closed__1; -lean_inc(x_98); -x_129 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_129, 0, x_98); -lean_ctor_set(x_129, 1, x_121); -lean_ctor_set(x_129, 2, x_128); -x_130 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; -lean_inc(x_98); +lean_ctor_set(x_120, 3, x_118); +x_121 = l_Lean_toolchain___closed__1; +lean_inc(x_105); +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_105); +lean_ctor_set(x_122, 1, x_121); +x_123 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__6; +lean_inc(x_106); +lean_inc(x_107); +x_124 = l_Lean_addMacroScope(x_107, x_123, x_106); +x_125 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__2; +x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__10; +lean_inc(x_105); +x_127 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_127, 0, x_105); +lean_ctor_set(x_127, 1, x_125); +lean_ctor_set(x_127, 2, x_124); +lean_ctor_set(x_127, 3, x_126); +x_128 = l_Lean_mkOptionalNode___closed__2; +lean_inc(x_105); +x_129 = l_Lean_Syntax_node1(x_105, x_128, x_127); +x_130 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; +lean_inc(x_105); x_131 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_131, 0, x_98); +lean_ctor_set(x_131, 0, x_105); lean_ctor_set(x_131, 1, x_130); -x_132 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; -lean_inc(x_98); -x_133 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_133, 0, x_98); -lean_ctor_set(x_133, 1, x_132); -lean_inc(x_98); -x_134 = l_Lean_Syntax_node1(x_98, x_121, x_113); -x_135 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; -lean_inc(x_98); -x_136 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_136, 0, x_98); -lean_ctor_set(x_136, 1, x_135); -lean_inc(x_98); -x_137 = l_Lean_Syntax_node2(x_98, x_121, x_134, x_136); -x_138 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; -lean_inc(x_99); -lean_inc(x_100); -x_139 = l_Lean_addMacroScope(x_100, x_138, x_99); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; -lean_inc(x_98); -x_141 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_141, 0, x_98); -lean_ctor_set(x_141, 1, x_140); -lean_ctor_set(x_141, 2, x_139); -lean_ctor_set(x_141, 3, x_111); -x_142 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; -lean_inc(x_129); -lean_inc(x_98); -x_143 = l_Lean_Syntax_node2(x_98, x_142, x_141, x_129); -x_144 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; -lean_inc(x_99); -lean_inc(x_100); -x_145 = l_Lean_addMacroScope(x_100, x_144, x_99); -x_146 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; -x_147 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; -lean_inc(x_98); +x_132 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; +lean_inc(x_131); +lean_inc(x_120); +lean_inc(x_109); +lean_inc(x_105); +x_133 = l_Lean_Syntax_node5(x_105, x_132, x_109, x_120, x_122, x_129, x_131); +lean_inc(x_105); +x_134 = l_Lean_Syntax_node1(x_105, x_128, x_133); +x_135 = l_Lean_mkSepArray___closed__1; +lean_inc(x_105); +x_136 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_136, 0, x_105); +lean_ctor_set(x_136, 1, x_128); +lean_ctor_set(x_136, 2, x_135); +x_137 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; +lean_inc(x_105); +x_138 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_138, 0, x_105); +lean_ctor_set(x_138, 1, x_137); +x_139 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; +lean_inc(x_105); +x_140 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_140, 0, x_105); +lean_ctor_set(x_140, 1, x_139); +lean_inc(x_105); +x_141 = l_Lean_Syntax_node1(x_105, x_128, x_120); +x_142 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; +lean_inc(x_105); +x_143 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_143, 0, x_105); +lean_ctor_set(x_143, 1, x_142); +lean_inc(x_105); +x_144 = l_Lean_Syntax_node2(x_105, x_128, x_141, x_143); +x_145 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; +lean_inc(x_106); +lean_inc(x_107); +x_146 = l_Lean_addMacroScope(x_107, x_145, x_106); +x_147 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; +lean_inc(x_105); x_148 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_148, 0, x_98); -lean_ctor_set(x_148, 1, x_146); -lean_ctor_set(x_148, 2, x_145); -lean_ctor_set(x_148, 3, x_147); -x_149 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; -lean_inc(x_148); +lean_ctor_set(x_148, 0, x_105); +lean_ctor_set(x_148, 1, x_147); +lean_ctor_set(x_148, 2, x_146); +lean_ctor_set(x_148, 3, x_118); +x_149 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; +lean_inc(x_136); +lean_inc(x_105); +x_150 = l_Lean_Syntax_node2(x_105, x_149, x_148, x_136); +x_151 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; lean_inc(x_106); -lean_inc(x_98); -x_150 = l_Lean_Syntax_node3(x_98, x_149, x_143, x_106, x_148); -x_151 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; -lean_inc(x_98); -x_152 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_152, 0, x_98); -lean_ctor_set(x_152, 1, x_151); -x_153 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; -x_154 = l_Lean_addMacroScope(x_100, x_153, x_99); -x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; -lean_inc(x_98); -x_156 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_156, 0, x_98); -lean_ctor_set(x_156, 1, x_155); -lean_ctor_set(x_156, 2, x_154); -lean_ctor_set(x_156, 3, x_111); -lean_inc(x_129); -lean_inc(x_98); -x_157 = l_Lean_Syntax_node2(x_98, x_142, x_156, x_129); +lean_inc(x_107); +x_152 = l_Lean_addMacroScope(x_107, x_151, x_106); +x_153 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; +x_154 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; +lean_inc(x_105); +x_155 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_155, 0, x_105); +lean_ctor_set(x_155, 1, x_153); +lean_ctor_set(x_155, 2, x_152); +lean_ctor_set(x_155, 3, x_154); +x_156 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_155); +lean_inc(x_113); +lean_inc(x_105); +x_157 = l_Lean_Syntax_node3(x_105, x_156, x_150, x_113, x_155); +x_158 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; +lean_inc(x_105); +x_159 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_159, 0, x_105); +lean_ctor_set(x_159, 1, x_158); +x_160 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; lean_inc(x_106); -lean_inc(x_98); -x_158 = l_Lean_Syntax_node3(x_98, x_149, x_157, x_106, x_148); -lean_inc(x_98); -x_159 = l_Lean_Syntax_node3(x_98, x_121, x_150, x_152, x_158); -x_160 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; -lean_inc(x_129); -lean_inc(x_98); -x_161 = l_Lean_Syntax_node1(x_98, x_160, x_129); -x_162 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; -lean_inc(x_98); -x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_98); +lean_inc(x_107); +x_161 = l_Lean_addMacroScope(x_107, x_160, x_106); +x_162 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; +lean_inc(x_105); +x_163 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_163, 0, x_105); lean_ctor_set(x_163, 1, x_162); -x_164 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_129); -lean_inc(x_98); -x_165 = l_Lean_Syntax_node6(x_98, x_164, x_133, x_137, x_159, x_161, x_129, x_163); -x_166 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; -lean_inc(x_98); -x_167 = l_Lean_Syntax_node4(x_98, x_166, x_127, x_129, x_131, x_165); -x_168 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; -lean_inc(x_98); -x_169 = l_Lean_Syntax_node2(x_98, x_168, x_108, x_167); -lean_inc(x_98); -x_170 = l_Lean_Syntax_node1(x_98, x_121, x_95); -x_171 = l_Lean_Syntax_mkApp___closed__2; -lean_inc(x_98); -x_172 = l_Lean_Syntax_node2(x_98, x_171, x_169, x_170); -x_173 = l_Lean_Syntax_node5(x_98, x_8, x_102, x_104, x_106, x_172, x_124); -x_174 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_173, x_2, x_3); +lean_ctor_set(x_163, 2, x_161); +lean_ctor_set(x_163, 3, x_118); +lean_inc(x_136); +lean_inc(x_105); +x_164 = l_Lean_Syntax_node2(x_105, x_149, x_163, x_136); +lean_inc(x_155); +lean_inc(x_113); +lean_inc(x_105); +x_165 = l_Lean_Syntax_node3(x_105, x_156, x_164, x_113, x_155); +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_167 = l_Lean_addMacroScope(x_107, x_166, x_106); +x_168 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_169 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_105); +x_170 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_170, 0, x_105); +lean_ctor_set(x_170, 1, x_168); +lean_ctor_set(x_170, 2, x_167); +lean_ctor_set(x_170, 3, x_169); +lean_inc(x_136); +lean_inc(x_105); +x_171 = l_Lean_Syntax_node2(x_105, x_149, x_170, x_136); +lean_inc(x_113); +lean_inc(x_105); +x_172 = l_Lean_Syntax_node3(x_105, x_156, x_171, x_113, x_155); +lean_inc(x_159); +lean_inc(x_105); +x_173 = l_Lean_Syntax_node5(x_105, x_128, x_157, x_159, x_165, x_159, x_172); +x_174 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +lean_inc(x_136); +lean_inc(x_105); +x_175 = l_Lean_Syntax_node1(x_105, x_174, x_136); +x_176 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_105); +x_177 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_177, 0, x_105); +lean_ctor_set(x_177, 1, x_176); +x_178 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_136); +lean_inc(x_105); +x_179 = l_Lean_Syntax_node6(x_105, x_178, x_140, x_144, x_173, x_175, x_136, x_177); +x_180 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +lean_inc(x_105); +x_181 = l_Lean_Syntax_node4(x_105, x_180, x_134, x_136, x_138, x_179); +x_182 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +lean_inc(x_105); +x_183 = l_Lean_Syntax_node2(x_105, x_182, x_115, x_181); +lean_inc(x_105); +x_184 = l_Lean_Syntax_node1(x_105, x_128, x_102); +x_185 = l_Lean_Syntax_mkApp___closed__2; +lean_inc(x_105); +x_186 = l_Lean_Syntax_node2(x_105, x_185, x_183, x_184); +x_187 = l_Lean_Syntax_node5(x_105, x_8, x_109, x_111, x_113, x_186, x_131); +x_188 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____lambda__1(x_1, x_187, x_2, x_3); lean_dec(x_2); -return x_174; +return x_188; } } } @@ -26457,7 +26621,7 @@ x_1 = l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__13; return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -26465,7 +26629,7 @@ x_1 = lean_mk_string_from_bytes("simp_all", 8); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -26473,7 +26637,7 @@ x_5 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tact x_6 = l_Lean_Syntax_setKind(x_1, x_5); x_7 = lean_unsigned_to_nat(0u); x_8 = l_Lean_Syntax_getArg(x_6, x_7); -x_9 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1; +x_9 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1; x_10 = 1; x_11 = l_Lean_mkAtomFrom(x_8, x_9, x_10); x_12 = l_Lean_Syntax_setArg(x_6, x_7, x_11); @@ -26493,7 +26657,7 @@ lean_ctor_set(x_20, 1, x_4); return x_20; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1() { _start: { lean_object* x_1; @@ -26501,16 +26665,16 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Simp.ConfigCtx", 24); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3() { _start: { lean_object* x_1; @@ -26518,65 +26682,65 @@ x_1 = lean_mk_string_from_bytes("ConfigCtx", 9); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__1; x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__3; x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__4; -x_4 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3; +x_4 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -26637,12 +26801,12 @@ lean_inc(x_12); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_12); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; lean_inc(x_13); lean_inc(x_14); x_31 = l_Lean_addMacroScope(x_14, x_30, x_13); -x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; lean_inc(x_12); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_12); @@ -26761,7 +26925,7 @@ x_82 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); x_83 = l_Lean_Syntax_node2(x_12, x_82, x_75, x_81); x_84 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_83, x_38); -x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_84, x_2, x_3); +x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_84, x_2, x_3); lean_dec(x_2); return x_85; } @@ -26816,12 +26980,12 @@ lean_inc(x_90); x_107 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_107, 0, x_90); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; lean_inc(x_91); lean_inc(x_92); x_109 = l_Lean_addMacroScope(x_92, x_108, x_91); -x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; +x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; lean_inc(x_90); x_112 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_112, 0, x_90); @@ -26925,17 +27089,17 @@ x_155 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_90); x_156 = l_Lean_Syntax_node2(x_90, x_155, x_153, x_154); x_157 = l_Lean_Syntax_node5(x_90, x_8, x_94, x_96, x_98, x_156, x_116); -x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_157, x_2, x_3); +x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_157, x_2, x_3); lean_dec(x_2); return x_158; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -27058,7 +27222,7 @@ x_1 = l_Lean_Parser_Tactic_simpAllArith___closed__9; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20025_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20209_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -27072,7 +27236,7 @@ lean_inc(x_7); x_9 = l_Lean_Syntax_isOfKind(x_7, x_8); if (x_9 == 0) { -lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_dec(x_7); x_10 = lean_ctor_get(x_2, 5); lean_inc(x_10); @@ -27119,12 +27283,12 @@ lean_inc(x_12); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_12); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; lean_inc(x_13); lean_inc(x_14); x_31 = l_Lean_addMacroScope(x_14, x_30, x_13); -x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; lean_inc(x_12); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_12); @@ -27188,6 +27352,8 @@ lean_inc(x_43); lean_inc(x_12); x_57 = l_Lean_Syntax_node2(x_12, x_56, x_55, x_43); x_58 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; +lean_inc(x_13); +lean_inc(x_14); x_59 = l_Lean_addMacroScope(x_14, x_58, x_13); x_60 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; x_61 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; @@ -27198,218 +27364,264 @@ lean_ctor_set(x_62, 1, x_60); lean_ctor_set(x_62, 2, x_59); lean_ctor_set(x_62, 3, x_61); x_63 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_62); lean_inc(x_20); lean_inc(x_12); x_64 = l_Lean_Syntax_node3(x_12, x_63, x_57, x_20, x_62); +x_65 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; lean_inc(x_12); -x_65 = l_Lean_Syntax_node1(x_12, x_35, x_64); -x_66 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +x_66 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_66, 0, x_12); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_68 = l_Lean_addMacroScope(x_14, x_67, x_13); +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_70 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_12); +x_71 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_71, 0, x_12); +lean_ctor_set(x_71, 1, x_69); +lean_ctor_set(x_71, 2, x_68); +lean_ctor_set(x_71, 3, x_70); lean_inc(x_43); lean_inc(x_12); -x_67 = l_Lean_Syntax_node1(x_12, x_66, x_43); -x_68 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +x_72 = l_Lean_Syntax_node2(x_12, x_56, x_71, x_43); +lean_inc(x_20); lean_inc(x_12); -x_69 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_69, 0, x_12); -lean_ctor_set(x_69, 1, x_68); -x_70 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_69); +x_73 = l_Lean_Syntax_node3(x_12, x_63, x_72, x_20, x_62); +lean_inc(x_12); +x_74 = l_Lean_Syntax_node3(x_12, x_35, x_64, x_66, x_73); +x_75 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; lean_inc(x_43); -lean_inc(x_67); +lean_inc(x_12); +x_76 = l_Lean_Syntax_node1(x_12, x_75, x_43); +x_77 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_12); +x_78 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_78, 0, x_12); +lean_ctor_set(x_78, 1, x_77); +x_79 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_78); +lean_inc(x_43); +lean_inc(x_76); lean_inc(x_47); lean_inc(x_12); -x_71 = l_Lean_Syntax_node6(x_12, x_70, x_47, x_51, x_65, x_67, x_43, x_69); -x_72 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +x_80 = l_Lean_Syntax_node6(x_12, x_79, x_47, x_51, x_74, x_76, x_43, x_78); +x_81 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; lean_inc(x_43); lean_inc(x_12); -x_73 = l_Lean_Syntax_node4(x_12, x_72, x_41, x_43, x_45, x_71); -x_74 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +x_82 = l_Lean_Syntax_node4(x_12, x_81, x_41, x_43, x_45, x_80); +x_83 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; lean_inc(x_12); -x_75 = l_Lean_Syntax_node2(x_12, x_74, x_22, x_73); -x_76 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; -lean_inc(x_69); +x_84 = l_Lean_Syntax_node2(x_12, x_83, x_22, x_82); +x_85 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; +lean_inc(x_78); lean_inc(x_47); lean_inc(x_12); -x_77 = l_Lean_Syntax_node2(x_12, x_76, x_47, x_69); +x_86 = l_Lean_Syntax_node2(x_12, x_85, x_47, x_78); lean_inc_n(x_43, 2); lean_inc(x_12); -x_78 = l_Lean_Syntax_node6(x_12, x_70, x_47, x_43, x_43, x_67, x_43, x_69); -x_79 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; +x_87 = l_Lean_Syntax_node6(x_12, x_79, x_47, x_43, x_43, x_76, x_43, x_78); +x_88 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; lean_inc(x_12); -x_80 = l_Lean_Syntax_node2(x_12, x_79, x_77, x_78); +x_89 = l_Lean_Syntax_node2(x_12, x_88, x_86, x_87); lean_inc(x_12); -x_81 = l_Lean_Syntax_node1(x_12, x_35, x_80); -x_82 = l_Lean_Syntax_mkApp___closed__2; +x_90 = l_Lean_Syntax_node1(x_12, x_35, x_89); +x_91 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); -x_83 = l_Lean_Syntax_node2(x_12, x_82, x_75, x_81); -x_84 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_83, x_38); -x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_84, x_2, x_3); +x_92 = l_Lean_Syntax_node2(x_12, x_91, x_84, x_90); +x_93 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_92, x_38); +x_94 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_93, x_2, x_3); lean_dec(x_2); -return x_85; +return x_94; } else -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t 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; -x_86 = lean_unsigned_to_nat(3u); -x_87 = l_Lean_Syntax_getArg(x_7, x_86); -lean_dec(x_7); -x_88 = lean_ctor_get(x_2, 5); -lean_inc(x_88); -x_89 = 0; -x_90 = l_Lean_SourceInfo_fromRef(x_88, x_89); -x_91 = lean_ctor_get(x_2, 2); -lean_inc(x_91); -x_92 = lean_ctor_get(x_2, 1); -lean_inc(x_92); -x_93 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; -lean_inc(x_90); -x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_90); -lean_ctor_set(x_94, 1, x_93); -x_95 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; -lean_inc(x_90); -x_96 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_96, 0, x_90); -lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; -lean_inc(x_90); -x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_90); -lean_ctor_set(x_98, 1, x_97); -x_99 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; -lean_inc(x_90); -x_100 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_100, 0, x_90); -lean_ctor_set(x_100, 1, x_99); -x_101 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; -lean_inc(x_91); -lean_inc(x_92); -x_102 = l_Lean_addMacroScope(x_92, x_101, x_91); -x_103 = lean_box(0); -x_104 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; -lean_inc(x_90); -x_105 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_105, 0, x_90); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_102); -lean_ctor_set(x_105, 3, x_103); -x_106 = l_Lean_toolchain___closed__1; -lean_inc(x_90); -x_107 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_107, 0, x_90); -lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; -lean_inc(x_91); -lean_inc(x_92); -x_109 = l_Lean_addMacroScope(x_92, x_108, x_91); -x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; -lean_inc(x_90); -x_112 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_112, 0, x_90); -lean_ctor_set(x_112, 1, x_110); -lean_ctor_set(x_112, 2, x_109); -lean_ctor_set(x_112, 3, x_111); -x_113 = l_Lean_mkOptionalNode___closed__2; -lean_inc(x_90); -x_114 = l_Lean_Syntax_node1(x_90, x_113, x_112); -x_115 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; -lean_inc(x_90); -x_116 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_116, 0, x_90); -lean_ctor_set(x_116, 1, x_115); -x_117 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; -lean_inc(x_116); -lean_inc(x_105); -lean_inc(x_94); -lean_inc(x_90); -x_118 = l_Lean_Syntax_node5(x_90, x_117, x_94, x_105, x_107, x_114, x_116); -lean_inc(x_90); -x_119 = l_Lean_Syntax_node1(x_90, x_113, x_118); -x_120 = l_Lean_mkSepArray___closed__1; -lean_inc(x_90); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_90); -lean_ctor_set(x_121, 1, x_113); -lean_ctor_set(x_121, 2, x_120); -x_122 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; -lean_inc(x_90); -x_123 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_123, 0, x_90); -lean_ctor_set(x_123, 1, x_122); -x_124 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; -lean_inc(x_90); +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; 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; +x_95 = lean_unsigned_to_nat(3u); +x_96 = l_Lean_Syntax_getArg(x_7, x_95); +lean_dec(x_7); +x_97 = lean_ctor_get(x_2, 5); +lean_inc(x_97); +x_98 = 0; +x_99 = l_Lean_SourceInfo_fromRef(x_97, x_98); +x_100 = lean_ctor_get(x_2, 2); +lean_inc(x_100); +x_101 = lean_ctor_get(x_2, 1); +lean_inc(x_101); +x_102 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; +lean_inc(x_99); +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_99); +lean_ctor_set(x_103, 1, x_102); +x_104 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; +lean_inc(x_99); +x_105 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_105, 0, x_99); +lean_ctor_set(x_105, 1, x_104); +x_106 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; +lean_inc(x_99); +x_107 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_107, 0, x_99); +lean_ctor_set(x_107, 1, x_106); +x_108 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; +lean_inc(x_99); +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_99); +lean_ctor_set(x_109, 1, x_108); +x_110 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; +lean_inc(x_100); +lean_inc(x_101); +x_111 = l_Lean_addMacroScope(x_101, x_110, x_100); +x_112 = lean_box(0); +x_113 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; +lean_inc(x_99); +x_114 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_114, 0, x_99); +lean_ctor_set(x_114, 1, x_113); +lean_ctor_set(x_114, 2, x_111); +lean_ctor_set(x_114, 3, x_112); +x_115 = l_Lean_toolchain___closed__1; +lean_inc(x_99); +x_116 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_116, 0, x_99); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; +lean_inc(x_100); +lean_inc(x_101); +x_118 = l_Lean_addMacroScope(x_101, x_117, x_100); +x_119 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_120 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; +lean_inc(x_99); +x_121 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_121, 0, x_99); +lean_ctor_set(x_121, 1, x_119); +lean_ctor_set(x_121, 2, x_118); +lean_ctor_set(x_121, 3, x_120); +x_122 = l_Lean_mkOptionalNode___closed__2; +lean_inc(x_99); +x_123 = l_Lean_Syntax_node1(x_99, x_122, x_121); +x_124 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; +lean_inc(x_99); x_125 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_125, 0, x_90); +lean_ctor_set(x_125, 0, x_99); lean_ctor_set(x_125, 1, x_124); -lean_inc(x_90); -x_126 = l_Lean_Syntax_node1(x_90, x_113, x_105); -x_127 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; -lean_inc(x_90); -x_128 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_128, 0, x_90); -lean_ctor_set(x_128, 1, x_127); -lean_inc(x_90); -x_129 = l_Lean_Syntax_node2(x_90, x_113, x_126, x_128); -x_130 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; -lean_inc(x_91); -lean_inc(x_92); -x_131 = l_Lean_addMacroScope(x_92, x_130, x_91); -x_132 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; -lean_inc(x_90); -x_133 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_133, 0, x_90); -lean_ctor_set(x_133, 1, x_132); -lean_ctor_set(x_133, 2, x_131); -lean_ctor_set(x_133, 3, x_103); -x_134 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; -lean_inc(x_121); -lean_inc(x_90); -x_135 = l_Lean_Syntax_node2(x_90, x_134, x_133, x_121); -x_136 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; -x_137 = l_Lean_addMacroScope(x_92, x_136, x_91); -x_138 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; -x_139 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; -lean_inc(x_90); -x_140 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_140, 0, x_90); -lean_ctor_set(x_140, 1, x_138); -lean_ctor_set(x_140, 2, x_137); -lean_ctor_set(x_140, 3, x_139); -x_141 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; -lean_inc(x_98); -lean_inc(x_90); -x_142 = l_Lean_Syntax_node3(x_90, x_141, x_135, x_98, x_140); -lean_inc(x_90); -x_143 = l_Lean_Syntax_node1(x_90, x_113, x_142); -x_144 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; -lean_inc(x_121); -lean_inc(x_90); -x_145 = l_Lean_Syntax_node1(x_90, x_144, x_121); -x_146 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; -lean_inc(x_90); -x_147 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_147, 0, x_90); -lean_ctor_set(x_147, 1, x_146); -x_148 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_121); -lean_inc(x_90); -x_149 = l_Lean_Syntax_node6(x_90, x_148, x_125, x_129, x_143, x_145, x_121, x_147); -x_150 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; -lean_inc(x_90); -x_151 = l_Lean_Syntax_node4(x_90, x_150, x_119, x_121, x_123, x_149); -x_152 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; -lean_inc(x_90); -x_153 = l_Lean_Syntax_node2(x_90, x_152, x_100, x_151); -lean_inc(x_90); -x_154 = l_Lean_Syntax_node1(x_90, x_113, x_87); -x_155 = l_Lean_Syntax_mkApp___closed__2; -lean_inc(x_90); -x_156 = l_Lean_Syntax_node2(x_90, x_155, x_153, x_154); -x_157 = l_Lean_Syntax_node5(x_90, x_8, x_94, x_96, x_98, x_156, x_116); -x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_157, x_2, x_3); +x_126 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; +lean_inc(x_125); +lean_inc(x_114); +lean_inc(x_103); +lean_inc(x_99); +x_127 = l_Lean_Syntax_node5(x_99, x_126, x_103, x_114, x_116, x_123, x_125); +lean_inc(x_99); +x_128 = l_Lean_Syntax_node1(x_99, x_122, x_127); +x_129 = l_Lean_mkSepArray___closed__1; +lean_inc(x_99); +x_130 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_130, 0, x_99); +lean_ctor_set(x_130, 1, x_122); +lean_ctor_set(x_130, 2, x_129); +x_131 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; +lean_inc(x_99); +x_132 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_132, 0, x_99); +lean_ctor_set(x_132, 1, x_131); +x_133 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; +lean_inc(x_99); +x_134 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_134, 0, x_99); +lean_ctor_set(x_134, 1, x_133); +lean_inc(x_99); +x_135 = l_Lean_Syntax_node1(x_99, x_122, x_114); +x_136 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; +lean_inc(x_99); +x_137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_137, 0, x_99); +lean_ctor_set(x_137, 1, x_136); +lean_inc(x_99); +x_138 = l_Lean_Syntax_node2(x_99, x_122, x_135, x_137); +x_139 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; +lean_inc(x_100); +lean_inc(x_101); +x_140 = l_Lean_addMacroScope(x_101, x_139, x_100); +x_141 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; +lean_inc(x_99); +x_142 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_142, 0, x_99); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +lean_ctor_set(x_142, 3, x_112); +x_143 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; +lean_inc(x_130); +lean_inc(x_99); +x_144 = l_Lean_Syntax_node2(x_99, x_143, x_142, x_130); +x_145 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; +lean_inc(x_100); +lean_inc(x_101); +x_146 = l_Lean_addMacroScope(x_101, x_145, x_100); +x_147 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; +x_148 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; +lean_inc(x_99); +x_149 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_149, 0, x_99); +lean_ctor_set(x_149, 1, x_147); +lean_ctor_set(x_149, 2, x_146); +lean_ctor_set(x_149, 3, x_148); +x_150 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_149); +lean_inc(x_107); +lean_inc(x_99); +x_151 = l_Lean_Syntax_node3(x_99, x_150, x_144, x_107, x_149); +x_152 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; +lean_inc(x_99); +x_153 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_153, 0, x_99); +lean_ctor_set(x_153, 1, x_152); +x_154 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_155 = l_Lean_addMacroScope(x_101, x_154, x_100); +x_156 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_157 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_99); +x_158 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_158, 0, x_99); +lean_ctor_set(x_158, 1, x_156); +lean_ctor_set(x_158, 2, x_155); +lean_ctor_set(x_158, 3, x_157); +lean_inc(x_130); +lean_inc(x_99); +x_159 = l_Lean_Syntax_node2(x_99, x_143, x_158, x_130); +lean_inc(x_107); +lean_inc(x_99); +x_160 = l_Lean_Syntax_node3(x_99, x_150, x_159, x_107, x_149); +lean_inc(x_99); +x_161 = l_Lean_Syntax_node3(x_99, x_122, x_151, x_153, x_160); +x_162 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +lean_inc(x_130); +lean_inc(x_99); +x_163 = l_Lean_Syntax_node1(x_99, x_162, x_130); +x_164 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_99); +x_165 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_165, 0, x_99); +lean_ctor_set(x_165, 1, x_164); +x_166 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_130); +lean_inc(x_99); +x_167 = l_Lean_Syntax_node6(x_99, x_166, x_134, x_138, x_161, x_163, x_130, x_165); +x_168 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +lean_inc(x_99); +x_169 = l_Lean_Syntax_node4(x_99, x_168, x_128, x_130, x_132, x_167); +x_170 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +lean_inc(x_99); +x_171 = l_Lean_Syntax_node2(x_99, x_170, x_109, x_169); +lean_inc(x_99); +x_172 = l_Lean_Syntax_node1(x_99, x_122, x_96); +x_173 = l_Lean_Syntax_mkApp___closed__2; +lean_inc(x_99); +x_174 = l_Lean_Syntax_node2(x_99, x_173, x_171, x_172); +x_175 = l_Lean_Syntax_node5(x_99, x_8, x_103, x_105, x_107, x_174, x_125); +x_176 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_175, x_2, x_3); lean_dec(x_2); -return x_158; +return x_176; } } } @@ -27531,7 +27743,7 @@ x_1 = l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__9; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20904_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21180_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -27545,7 +27757,7 @@ lean_inc(x_7); x_9 = l_Lean_Syntax_isOfKind(x_7, x_8); if (x_9 == 0) { -lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_dec(x_7); x_10 = lean_ctor_get(x_2, 5); lean_inc(x_10); @@ -27592,12 +27804,12 @@ lean_inc(x_12); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_12); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; lean_inc(x_13); lean_inc(x_14); x_31 = l_Lean_addMacroScope(x_14, x_30, x_13); -x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; lean_inc(x_12); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_12); @@ -27683,6 +27895,8 @@ x_66 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_66, 0, x_12); lean_ctor_set(x_66, 1, x_65); x_67 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; +lean_inc(x_13); +lean_inc(x_14); x_68 = l_Lean_addMacroScope(x_14, x_67, x_13); x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; lean_inc(x_12); @@ -27694,241 +27908,279 @@ lean_ctor_set(x_70, 3, x_25); lean_inc(x_43); lean_inc(x_12); x_71 = l_Lean_Syntax_node2(x_12, x_56, x_70, x_43); +lean_inc(x_62); lean_inc(x_20); lean_inc(x_12); x_72 = l_Lean_Syntax_node3(x_12, x_63, x_71, x_20, x_62); +x_73 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_74 = l_Lean_addMacroScope(x_14, x_73, x_13); +x_75 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_76 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; lean_inc(x_12); -x_73 = l_Lean_Syntax_node3(x_12, x_35, x_64, x_66, x_72); -x_74 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +x_77 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_77, 0, x_12); +lean_ctor_set(x_77, 1, x_75); +lean_ctor_set(x_77, 2, x_74); +lean_ctor_set(x_77, 3, x_76); lean_inc(x_43); lean_inc(x_12); -x_75 = l_Lean_Syntax_node1(x_12, x_74, x_43); -x_76 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +x_78 = l_Lean_Syntax_node2(x_12, x_56, x_77, x_43); +lean_inc(x_20); lean_inc(x_12); -x_77 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_77, 0, x_12); -lean_ctor_set(x_77, 1, x_76); -x_78 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_77); +x_79 = l_Lean_Syntax_node3(x_12, x_63, x_78, x_20, x_62); +lean_inc(x_66); +lean_inc(x_12); +x_80 = l_Lean_Syntax_node5(x_12, x_35, x_64, x_66, x_72, x_66, x_79); +x_81 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; lean_inc(x_43); -lean_inc(x_75); +lean_inc(x_12); +x_82 = l_Lean_Syntax_node1(x_12, x_81, x_43); +x_83 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_12); +x_84 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_84, 0, x_12); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_84); +lean_inc(x_43); +lean_inc(x_82); lean_inc(x_47); lean_inc(x_12); -x_79 = l_Lean_Syntax_node6(x_12, x_78, x_47, x_51, x_73, x_75, x_43, x_77); -x_80 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +x_86 = l_Lean_Syntax_node6(x_12, x_85, x_47, x_51, x_80, x_82, x_43, x_84); +x_87 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; lean_inc(x_43); lean_inc(x_12); -x_81 = l_Lean_Syntax_node4(x_12, x_80, x_41, x_43, x_45, x_79); -x_82 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +x_88 = l_Lean_Syntax_node4(x_12, x_87, x_41, x_43, x_45, x_86); +x_89 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; lean_inc(x_12); -x_83 = l_Lean_Syntax_node2(x_12, x_82, x_22, x_81); -x_84 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; -lean_inc(x_77); +x_90 = l_Lean_Syntax_node2(x_12, x_89, x_22, x_88); +x_91 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__90; +lean_inc(x_84); lean_inc(x_47); lean_inc(x_12); -x_85 = l_Lean_Syntax_node2(x_12, x_84, x_47, x_77); +x_92 = l_Lean_Syntax_node2(x_12, x_91, x_47, x_84); lean_inc_n(x_43, 2); lean_inc(x_12); -x_86 = l_Lean_Syntax_node6(x_12, x_78, x_47, x_43, x_43, x_75, x_43, x_77); -x_87 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; +x_93 = l_Lean_Syntax_node6(x_12, x_85, x_47, x_43, x_43, x_82, x_43, x_84); +x_94 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__88; lean_inc(x_12); -x_88 = l_Lean_Syntax_node2(x_12, x_87, x_85, x_86); +x_95 = l_Lean_Syntax_node2(x_12, x_94, x_92, x_93); lean_inc(x_12); -x_89 = l_Lean_Syntax_node1(x_12, x_35, x_88); -x_90 = l_Lean_Syntax_mkApp___closed__2; +x_96 = l_Lean_Syntax_node1(x_12, x_35, x_95); +x_97 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); -x_91 = l_Lean_Syntax_node2(x_12, x_90, x_83, x_89); -x_92 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_91, x_38); -x_93 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_92, x_2, x_3); +x_98 = l_Lean_Syntax_node2(x_12, x_97, x_90, x_96); +x_99 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_98, x_38); +x_100 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_99, x_2, x_3); lean_dec(x_2); -return x_93; +return x_100; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; 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; -x_94 = lean_unsigned_to_nat(3u); -x_95 = l_Lean_Syntax_getArg(x_7, x_94); +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; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; +x_101 = lean_unsigned_to_nat(3u); +x_102 = l_Lean_Syntax_getArg(x_7, x_101); lean_dec(x_7); -x_96 = lean_ctor_get(x_2, 5); -lean_inc(x_96); -x_97 = 0; -x_98 = l_Lean_SourceInfo_fromRef(x_96, x_97); -x_99 = lean_ctor_get(x_2, 2); -lean_inc(x_99); -x_100 = lean_ctor_get(x_2, 1); -lean_inc(x_100); -x_101 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; -lean_inc(x_98); -x_102 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_102, 0, x_98); -lean_ctor_set(x_102, 1, x_101); -x_103 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; -lean_inc(x_98); -x_104 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_104, 0, x_98); -lean_ctor_set(x_104, 1, x_103); -x_105 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; -lean_inc(x_98); -x_106 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_106, 0, x_98); -lean_ctor_set(x_106, 1, x_105); -x_107 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; -lean_inc(x_98); -x_108 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_108, 0, x_98); -lean_ctor_set(x_108, 1, x_107); -x_109 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; -lean_inc(x_99); -lean_inc(x_100); -x_110 = l_Lean_addMacroScope(x_100, x_109, x_99); -x_111 = lean_box(0); -x_112 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; -lean_inc(x_98); -x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_98); +x_103 = lean_ctor_get(x_2, 5); +lean_inc(x_103); +x_104 = 0; +x_105 = l_Lean_SourceInfo_fromRef(x_103, x_104); +x_106 = lean_ctor_get(x_2, 2); +lean_inc(x_106); +x_107 = lean_ctor_get(x_2, 1); +lean_inc(x_107); +x_108 = l_Lean_TSyntax_expandInterpolatedStr___closed__4; +lean_inc(x_105); +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_105); +lean_ctor_set(x_109, 1, x_108); +x_110 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__4; +lean_inc(x_105); +x_111 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_111, 0, x_105); +lean_ctor_set(x_111, 1, x_110); +x_112 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; +lean_inc(x_105); +x_113 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_113, 0, x_105); lean_ctor_set(x_113, 1, x_112); -lean_ctor_set(x_113, 2, x_110); -lean_ctor_set(x_113, 3, x_111); -x_114 = l_Lean_toolchain___closed__1; -lean_inc(x_98); +x_114 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__34; +lean_inc(x_105); x_115 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_115, 0, x_98); +lean_ctor_set(x_115, 0, x_105); lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4; -lean_inc(x_99); -lean_inc(x_100); -x_117 = l_Lean_addMacroScope(x_100, x_116, x_99); -x_118 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2; -x_119 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8; -lean_inc(x_98); +x_116 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__55; +lean_inc(x_106); +lean_inc(x_107); +x_117 = l_Lean_addMacroScope(x_107, x_116, x_106); +x_118 = lean_box(0); +x_119 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__54; +lean_inc(x_105); x_120 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_120, 0, x_98); -lean_ctor_set(x_120, 1, x_118); +lean_ctor_set(x_120, 0, x_105); +lean_ctor_set(x_120, 1, x_119); lean_ctor_set(x_120, 2, x_117); -lean_ctor_set(x_120, 3, x_119); -x_121 = l_Lean_mkOptionalNode___closed__2; -lean_inc(x_98); -x_122 = l_Lean_Syntax_node1(x_98, x_121, x_120); -x_123 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; -lean_inc(x_98); -x_124 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_124, 0, x_98); -lean_ctor_set(x_124, 1, x_123); -x_125 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; -lean_inc(x_124); -lean_inc(x_113); -lean_inc(x_102); -lean_inc(x_98); -x_126 = l_Lean_Syntax_node5(x_98, x_125, x_102, x_113, x_115, x_122, x_124); -lean_inc(x_98); -x_127 = l_Lean_Syntax_node1(x_98, x_121, x_126); -x_128 = l_Lean_mkSepArray___closed__1; -lean_inc(x_98); -x_129 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_129, 0, x_98); -lean_ctor_set(x_129, 1, x_121); -lean_ctor_set(x_129, 2, x_128); -x_130 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; -lean_inc(x_98); +lean_ctor_set(x_120, 3, x_118); +x_121 = l_Lean_toolchain___closed__1; +lean_inc(x_105); +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_105); +lean_ctor_set(x_122, 1, x_121); +x_123 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4; +lean_inc(x_106); +lean_inc(x_107); +x_124 = l_Lean_addMacroScope(x_107, x_123, x_106); +x_125 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2; +x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8; +lean_inc(x_105); +x_127 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_127, 0, x_105); +lean_ctor_set(x_127, 1, x_125); +lean_ctor_set(x_127, 2, x_124); +lean_ctor_set(x_127, 3, x_126); +x_128 = l_Lean_mkOptionalNode___closed__2; +lean_inc(x_105); +x_129 = l_Lean_Syntax_node1(x_105, x_128, x_127); +x_130 = l_Lean_TSyntax_expandInterpolatedStr___closed__5; +lean_inc(x_105); x_131 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_131, 0, x_98); +lean_ctor_set(x_131, 0, x_105); lean_ctor_set(x_131, 1, x_130); -x_132 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; -lean_inc(x_98); -x_133 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_133, 0, x_98); -lean_ctor_set(x_133, 1, x_132); -lean_inc(x_98); -x_134 = l_Lean_Syntax_node1(x_98, x_121, x_113); -x_135 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; -lean_inc(x_98); -x_136 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_136, 0, x_98); -lean_ctor_set(x_136, 1, x_135); -lean_inc(x_98); -x_137 = l_Lean_Syntax_node2(x_98, x_121, x_134, x_136); -x_138 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; -lean_inc(x_99); -lean_inc(x_100); -x_139 = l_Lean_addMacroScope(x_100, x_138, x_99); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; -lean_inc(x_98); -x_141 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_141, 0, x_98); -lean_ctor_set(x_141, 1, x_140); -lean_ctor_set(x_141, 2, x_139); -lean_ctor_set(x_141, 3, x_111); -x_142 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; -lean_inc(x_129); -lean_inc(x_98); -x_143 = l_Lean_Syntax_node2(x_98, x_142, x_141, x_129); -x_144 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; -lean_inc(x_99); -lean_inc(x_100); -x_145 = l_Lean_addMacroScope(x_100, x_144, x_99); -x_146 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; -x_147 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; -lean_inc(x_98); +x_132 = l_Lean_TSyntax_expandInterpolatedStr___closed__3; +lean_inc(x_131); +lean_inc(x_120); +lean_inc(x_109); +lean_inc(x_105); +x_133 = l_Lean_Syntax_node5(x_105, x_132, x_109, x_120, x_122, x_129, x_131); +lean_inc(x_105); +x_134 = l_Lean_Syntax_node1(x_105, x_128, x_133); +x_135 = l_Lean_mkSepArray___closed__1; +lean_inc(x_105); +x_136 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_136, 0, x_105); +lean_ctor_set(x_136, 1, x_128); +lean_ctor_set(x_136, 2, x_135); +x_137 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__41; +lean_inc(x_105); +x_138 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_138, 0, x_105); +lean_ctor_set(x_138, 1, x_137); +x_139 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; +lean_inc(x_105); +x_140 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_140, 0, x_105); +lean_ctor_set(x_140, 1, x_139); +lean_inc(x_105); +x_141 = l_Lean_Syntax_node1(x_105, x_128, x_120); +x_142 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__66; +lean_inc(x_105); +x_143 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_143, 0, x_105); +lean_ctor_set(x_143, 1, x_142); +lean_inc(x_105); +x_144 = l_Lean_Syntax_node2(x_105, x_128, x_141, x_143); +x_145 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3; +lean_inc(x_106); +lean_inc(x_107); +x_146 = l_Lean_addMacroScope(x_107, x_145, x_106); +x_147 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2; +lean_inc(x_105); x_148 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_148, 0, x_98); -lean_ctor_set(x_148, 1, x_146); -lean_ctor_set(x_148, 2, x_145); -lean_ctor_set(x_148, 3, x_147); -x_149 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; -lean_inc(x_148); +lean_ctor_set(x_148, 0, x_105); +lean_ctor_set(x_148, 1, x_147); +lean_ctor_set(x_148, 2, x_146); +lean_ctor_set(x_148, 3, x_118); +x_149 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; +lean_inc(x_136); +lean_inc(x_105); +x_150 = l_Lean_Syntax_node2(x_105, x_149, x_148, x_136); +x_151 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__121; lean_inc(x_106); -lean_inc(x_98); -x_150 = l_Lean_Syntax_node3(x_98, x_149, x_143, x_106, x_148); -x_151 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; -lean_inc(x_98); -x_152 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_152, 0, x_98); -lean_ctor_set(x_152, 1, x_151); -x_153 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; -x_154 = l_Lean_addMacroScope(x_100, x_153, x_99); -x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; -lean_inc(x_98); -x_156 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_156, 0, x_98); -lean_ctor_set(x_156, 1, x_155); -lean_ctor_set(x_156, 2, x_154); -lean_ctor_set(x_156, 3, x_111); -lean_inc(x_129); -lean_inc(x_98); -x_157 = l_Lean_Syntax_node2(x_98, x_142, x_156, x_129); +lean_inc(x_107); +x_152 = l_Lean_addMacroScope(x_107, x_151, x_106); +x_153 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__120; +x_154 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__123; +lean_inc(x_105); +x_155 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_155, 0, x_105); +lean_ctor_set(x_155, 1, x_153); +lean_ctor_set(x_155, 2, x_152); +lean_ctor_set(x_155, 3, x_154); +x_156 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__11; +lean_inc(x_155); +lean_inc(x_113); +lean_inc(x_105); +x_157 = l_Lean_Syntax_node3(x_105, x_156, x_150, x_113, x_155); +x_158 = l_List_repr_x27___at___private_Init_Meta_0__Lean_Syntax_reprPreresolved____x40_Init_Meta___hyg_2212____spec__1___closed__3; +lean_inc(x_105); +x_159 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_159, 0, x_105); +lean_ctor_set(x_159, 1, x_158); +x_160 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__13; lean_inc(x_106); -lean_inc(x_98); -x_158 = l_Lean_Syntax_node3(x_98, x_149, x_157, x_106, x_148); -lean_inc(x_98); -x_159 = l_Lean_Syntax_node3(x_98, x_121, x_150, x_152, x_158); -x_160 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; -lean_inc(x_129); -lean_inc(x_98); -x_161 = l_Lean_Syntax_node1(x_98, x_160, x_129); -x_162 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; -lean_inc(x_98); -x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_98); +lean_inc(x_107); +x_161 = l_Lean_addMacroScope(x_107, x_160, x_106); +x_162 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__12; +lean_inc(x_105); +x_163 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_163, 0, x_105); lean_ctor_set(x_163, 1, x_162); -x_164 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; -lean_inc(x_129); -lean_inc(x_98); -x_165 = l_Lean_Syntax_node6(x_98, x_164, x_133, x_137, x_159, x_161, x_129, x_163); -x_166 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; -lean_inc(x_98); -x_167 = l_Lean_Syntax_node4(x_98, x_166, x_127, x_129, x_131, x_165); -x_168 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; -lean_inc(x_98); -x_169 = l_Lean_Syntax_node2(x_98, x_168, x_108, x_167); -lean_inc(x_98); -x_170 = l_Lean_Syntax_node1(x_98, x_121, x_95); -x_171 = l_Lean_Syntax_mkApp___closed__2; -lean_inc(x_98); -x_172 = l_Lean_Syntax_node2(x_98, x_171, x_169, x_170); -x_173 = l_Lean_Syntax_node5(x_98, x_8, x_102, x_104, x_106, x_172, x_124); -x_174 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1(x_1, x_173, x_2, x_3); +lean_ctor_set(x_163, 2, x_161); +lean_ctor_set(x_163, 3, x_118); +lean_inc(x_136); +lean_inc(x_105); +x_164 = l_Lean_Syntax_node2(x_105, x_149, x_163, x_136); +lean_inc(x_155); +lean_inc(x_113); +lean_inc(x_105); +x_165 = l_Lean_Syntax_node3(x_105, x_156, x_164, x_113, x_155); +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6; +x_167 = l_Lean_addMacroScope(x_107, x_166, x_106); +x_168 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5; +x_169 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10; +lean_inc(x_105); +x_170 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_170, 0, x_105); +lean_ctor_set(x_170, 1, x_168); +lean_ctor_set(x_170, 2, x_167); +lean_ctor_set(x_170, 3, x_169); +lean_inc(x_136); +lean_inc(x_105); +x_171 = l_Lean_Syntax_node2(x_105, x_149, x_170, x_136); +lean_inc(x_113); +lean_inc(x_105); +x_172 = l_Lean_Syntax_node3(x_105, x_156, x_171, x_113, x_155); +lean_inc(x_159); +lean_inc(x_105); +x_173 = l_Lean_Syntax_node5(x_105, x_128, x_157, x_159, x_165, x_159, x_172); +x_174 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__29; +lean_inc(x_136); +lean_inc(x_105); +x_175 = l_Lean_Syntax_node1(x_105, x_174, x_136); +x_176 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; +lean_inc(x_105); +x_177 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_177, 0, x_105); +lean_ctor_set(x_177, 1, x_176); +x_178 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__8; +lean_inc(x_136); +lean_inc(x_105); +x_179 = l_Lean_Syntax_node6(x_105, x_178, x_140, x_144, x_173, x_175, x_136, x_177); +x_180 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__37; +lean_inc(x_105); +x_181 = l_Lean_Syntax_node4(x_105, x_180, x_134, x_136, x_138, x_179); +x_182 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__declareSimpLikeTactic__1___lambda__1___closed__35; +lean_inc(x_105); +x_183 = l_Lean_Syntax_node2(x_105, x_182, x_115, x_181); +lean_inc(x_105); +x_184 = l_Lean_Syntax_node1(x_105, x_128, x_102); +x_185 = l_Lean_Syntax_mkApp___closed__2; +lean_inc(x_105); +x_186 = l_Lean_Syntax_node2(x_105, x_185, x_183, x_184); +x_187 = l_Lean_Syntax_node5(x_105, x_8, x_109, x_111, x_113, x_186, x_131); +x_188 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1(x_1, x_187, x_2, x_3); lean_dec(x_2); -return x_174; +return x_188; } } } @@ -28064,7 +28316,7 @@ x_1 = l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__10; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -28092,7 +28344,7 @@ lean_ctor_set(x_20, 1, x_4); return x_20; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1() { _start: { lean_object* x_1; @@ -28100,16 +28352,16 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.DSimp.Config", 22); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3() { _start: { lean_object* x_1; @@ -28117,65 +28369,65 @@ x_1 = lean_mk_string_from_bytes("DSimp", 5); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__1; x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__3; -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3; x_4 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16391____closed__5; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -28236,12 +28488,12 @@ lean_inc(x_12); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_12); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4; lean_inc(x_13); lean_inc(x_14); x_31 = l_Lean_addMacroScope(x_14, x_30, x_13); -x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8; lean_inc(x_12); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_12); @@ -28360,7 +28612,7 @@ x_82 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_12); x_83 = l_Lean_Syntax_node2(x_12, x_82, x_75, x_81); x_84 = l_Lean_Syntax_node5(x_12, x_8, x_16, x_18, x_20, x_83, x_38); -x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1(x_1, x_84, x_2, x_3); +x_85 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1(x_1, x_84, x_2, x_3); lean_dec(x_2); return x_85; } @@ -28415,12 +28667,12 @@ lean_inc(x_90); x_107 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_107, 0, x_90); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4; +x_108 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4; lean_inc(x_91); lean_inc(x_92); x_109 = l_Lean_addMacroScope(x_92, x_108, x_91); -x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2; -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8; +x_110 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8; lean_inc(x_90); x_112 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_112, 0, x_90); @@ -28524,17 +28776,17 @@ x_155 = l_Lean_Syntax_mkApp___closed__2; lean_inc(x_90); x_156 = l_Lean_Syntax_node2(x_90, x_155, x_153, x_154); x_157 = l_Lean_Syntax_node5(x_90, x_8, x_94, x_96, x_98, x_156, x_116); -x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1(x_1, x_157, x_2, x_3); +x_158 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1(x_1, x_157, x_2, x_3); lean_dec(x_2); return x_158; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -29946,6 +30198,20 @@ l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2 = _ini lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__2); l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__8); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__9); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17284____closed__10); l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__1 = _init_l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__1); l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__2 = _init_l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__2(); @@ -29996,24 +30262,24 @@ l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__13 = _init_l_Lean_Parser_Tactic lean_mark_persistent(l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__13); l_Lean_Parser_Tactic_simpAllAutoUnfold = _init_l_Lean_Parser_Tactic_simpAllAutoUnfold(); lean_mark_persistent(l_Lean_Parser_Tactic_simpAllAutoUnfold); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____lambda__1___closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__3); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__4); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__5); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__6); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__7); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19146____closed__8); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____lambda__1___closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19330____closed__8); l_Lean_Parser_Tactic_simpAllArith___closed__1 = _init_l_Lean_Parser_Tactic_simpAllArith___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_simpAllArith___closed__1); l_Lean_Parser_Tactic_simpAllArith___closed__2 = _init_l_Lean_Parser_Tactic_simpAllArith___closed__2(); @@ -30076,22 +30342,22 @@ l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__10 = _init_l_Lean_Parser_Tactic_d lean_mark_persistent(l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__10); l_Lean_Parser_Tactic_dsimpAutoUnfold = _init_l_Lean_Parser_Tactic_dsimpAutoUnfold(); lean_mark_persistent(l_Lean_Parser_Tactic_dsimpAutoUnfold); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__3); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__4); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__5); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__6); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__7); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21867____closed__8); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_22235____closed__8); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/MetaTypes.c b/stage0/stdlib/Init/MetaTypes.c index 5546eb6db1e5..831271540ce3 100644 --- a/stage0/stdlib/Init/MetaTypes.c +++ b/stage0/stdlib/Init/MetaTypes.c @@ -993,7 +993,7 @@ static uint8_t _init_l_Lean_Meta_Simp_Config_decide___default() { _start: { uint8_t x_1; -x_1 = 1; +x_1 = 0; return x_1; } } diff --git a/stage0/stdlib/Lean/Compiler/LCNF/AuxDeclCache.c b/stage0/stdlib/Lean/Compiler/LCNF/AuxDeclCache.c index 09cb55bddb23..91429ffa816a 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/AuxDeclCache.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/AuxDeclCache.c @@ -25,7 +25,6 @@ size_t lean_usize_mul(size_t, size_t); lean_object* l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(lean_object*, lean_object*); lean_object* l_Lean_EnvExtension_modifyState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_AuxDeclCache___hyg_9____closed__3; lean_object* l_Lean_EnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); @@ -43,6 +42,7 @@ static lean_object* l_Lean_Compiler_LCNF_cacheAuxDecl___closed__4; static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_AuxDeclCache___hyg_9____closed__4; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_cacheAuxDecl___lambda__1(lean_object*, lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Compiler_LCNF_cacheAuxDecl___spec__2___closed__2; +uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(lean_object*, lean_object*); extern lean_object* l_Lean_Compiler_LCNF_instBEqDecl; static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_AuxDeclCache___hyg_9____closed__1; lean_object* lean_usize_to_nat(size_t); @@ -142,7 +142,7 @@ else lean_object* x_9; uint8_t x_10; x_9 = lean_array_fget(x_1, x_4); lean_inc(x_5); -x_10 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_5, x_9); +x_10 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_5, x_9); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; @@ -212,7 +212,7 @@ lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_3, x_11); +x_13 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_3, x_11); if (x_13 == 0) { lean_object* x_14; @@ -360,7 +360,7 @@ else lean_object* x_17; uint8_t x_18; x_17 = lean_array_fget(x_5, x_2); lean_inc(x_3); -x_18 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_3, x_17); +x_18 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_3, x_17); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; @@ -458,7 +458,7 @@ x_19 = lean_ctor_get(x_15, 0); x_20 = lean_ctor_get(x_15, 1); lean_inc(x_19); lean_inc(x_4); -x_21 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_4, x_19); +x_21 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_4, x_19); if (x_21 == 0) { lean_object* x_22; lean_object* x_23; lean_object* x_24; @@ -494,7 +494,7 @@ lean_inc(x_26); lean_dec(x_15); lean_inc(x_26); lean_inc(x_4); -x_28 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_4, x_26); +x_28 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_4, x_26); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; @@ -617,7 +617,7 @@ if (lean_is_exclusive(x_57)) { } lean_inc(x_60); lean_inc(x_4); -x_63 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_4, x_60); +x_63 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_4, x_60); if (x_63 == 0) { lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Basic.c b/stage0/stdlib/Lean/Compiler/LCNF/Basic.c index ffa9ede1bc5a..ce1b7261f9ad 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Basic.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Basic.c @@ -44,6 +44,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_e uint8_t l___private_Lean_Compiler_InlineAttrs_0__Lean_Compiler_beqInlineAttributeKind____x40_Lean_Compiler_InlineAttrs___hyg_23_(uint8_t, uint8_t); lean_object* l_Lean_Level_instantiateParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instInhabitedLetValue; +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Code_forM_go___spec__1(lean_object*); uint64_t lean_uint64_of_nat(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); @@ -54,7 +55,6 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_attachCodeDecls_go(lean_object*, l LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instInhabitedFunDeclCore___rarg(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateFunImp___closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_collectUsedAtExpr(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateAltsImp___spec__1(lean_object*); lean_object* l_Lean_Expr_lit___override(lean_object*); static lean_object* l_Lean_Compiler_LCNF_instInhabitedCasesCore___closed__1; @@ -79,7 +79,6 @@ lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Code_size_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Arg_toLetValue(lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instInhabitedAltCore___rarg(lean_object*); static lean_object* l_Lean_Compiler_LCNF_CasesCore_extractAlt_x21___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_hashArg____x40_Lean_Compiler_LCNF_Basic___hyg_630____boxed(lean_object*); @@ -95,6 +94,7 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Code_forM_go___rarg(lean_object*, LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqAlt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instInhabitedAltCore(lean_object*); static lean_object* l_Lean_Compiler_LCNF_instInhabitedLetDecl___closed__1; +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateJmpImp___closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_AltCore_forCodeM(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); @@ -108,7 +108,6 @@ static lean_object* l_Lean_Compiler_LCNF_instBEqFunDecl___closed__1; LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_CasesCore_extractAlt_x21___lambda__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqCases___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Compiler_LCNF_markRecDecls_visit___spec__1(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1(lean_object*, lean_object*); size_t lean_ptr_addr(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateReturnImp___closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Code_forM_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -143,10 +142,10 @@ static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_u LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_markRecDecls_go(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqCases(lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_LetValue_updateConstImp___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_instInhabitedCodeDecl___closed__1; LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqCases___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Param_toArg(lean_object*); -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_collectParams___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_Code_sizeLe(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_collectType___spec__1___lambda__1(lean_object*); @@ -161,7 +160,6 @@ uint8_t l_Lean_Compiler_hasSpecializeAttribute(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_markRecDecls_visit___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_Decl_inlineable(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateCasesImp___closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Decl_alwaysInlineAttr___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_instantiateRangeArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -188,6 +186,7 @@ uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instHashableArg; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_LitValue_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_collectParams___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_markRecDecls(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instBEqParam; LEAN_EXPORT uint64_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_hashLetValue____x40_Lean_Compiler_LCNF_Basic___hyg_1241_(lean_object*); @@ -248,6 +247,7 @@ static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_u LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqCases___boxed(lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Compiler_LCNF_CasesCore_extractAlt_x21___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instantiateRangeArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instantiateRevRangeArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Decl_isCasesOnParam_x3f(lean_object*); @@ -278,7 +278,6 @@ uint64_t l_Lean_Name_hash___override(lean_object*); LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_eqImp___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Arg_toExpr(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_Arg_updateTypeImp___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_CodeDecl_fvarId(lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); uint64_t l_List_foldl___at_Lean_Expr_const___override___spec__1(uint64_t, lean_object*); @@ -372,6 +371,7 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_hasLocalInst___boxed(lean_object*) LEAN_EXPORT lean_object* l_panic___at_Lean_Compiler_LCNF_CasesCore_extractAlt_x21___spec__1(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateCasesImp___closed__1; LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_Decl_isCasesOnParam_x3f_go___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_Compiler_LCNF_instInhabitedParam___closed__1() { _start: { @@ -6675,7 +6675,7 @@ x_1 = l_Lean_Compiler_LCNF_instInhabitedDecl___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -6722,7 +6722,7 @@ return x_10; } } } -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -6764,7 +6764,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; 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; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; uint8_t x_25; @@ -6879,7 +6879,7 @@ else { lean_object* x_35; uint8_t x_36; x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2(x_6, x_14, lean_box(0), x_6, x_14, x_35); +x_36 = l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2(x_6, x_14, lean_box(0), x_6, x_14, x_35); lean_dec(x_14); lean_dec(x_6); if (x_36 == 0) @@ -6957,7 +6957,7 @@ if (x_9 == 0) if (x_17 == 0) { uint8_t x_20; -x_20 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1(x_10, x_18); +x_20 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1(x_10, x_18); return x_20; } else @@ -6982,27 +6982,27 @@ return x_22; else { uint8_t x_23; -x_23 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1(x_10, x_18); +x_23 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1(x_10, x_18); return x_23; } } } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__1(x_1, x_2); +x_3 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_1119____at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__1(x_1, x_2); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; -x_7 = l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____spec__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_isEqvAux___at___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____spec__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -7011,11 +7011,11 @@ x_8 = lean_box(x_7); return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_1, x_2); +x_3 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_1, x_2); x_4 = lean_box(x_3); return x_4; } @@ -7024,7 +7024,7 @@ static lean_object* _init_l_Lean_Compiler_LCNF_instBEqDecl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796____boxed), 2, 0); return x_1; } } diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Simp/JpCases.c b/stage0/stdlib/Lean/Compiler/LCNF/Simp/JpCases.c index 6932211f841a..c8dc34728b07 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Simp/JpCases.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Simp/JpCases.c @@ -16,7 +16,6 @@ extern "C" { lean_object* l_Lean_Compiler_LCNF_mkAuxLetDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJmp_x3f___spec__2(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__outOfBounds___rarg(lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10; LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJmp_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Compiler_LCNF_Simp_collectJpCasesInfo_go___spec__1(lean_object*, lean_object*); @@ -29,8 +28,9 @@ static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___clos lean_object* l_Lean_Compiler_LCNF_Internalize_internalizeCode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_isJpCases_x3f_go(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJmp_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6; static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJmp_x3f___closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_any___at_Lean_Compiler_LCNF_Simp_JpCasesInfoMap_isCandidate___spec__1___boxed(lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Simp_withDiscrCtorImp_updateCtx___spec__5(size_t, size_t, lean_object*); @@ -49,8 +49,8 @@ lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJmpNewArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12; LEAN_EXPORT lean_object* l_Lean_RBNode_revFold___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__2___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4; uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT uint8_t l_Lean_RBNode_any___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -72,20 +72,22 @@ static lean_object* l_List_forIn_loop___at_Lean_Compiler_LCNF_Simp_simpJpCases_x lean_object* l_Lean_stringToMessageData(lean_object*); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6; lean_object* l_Lean_Compiler_LCNF_LCtx_toLocalContext(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___closed__2; LEAN_EXPORT lean_object* l_Lean_RBNode_revFold___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__4(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7; static lean_object* l_List_forIn_loop___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__7___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_ptr_addr(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_extractJpCases_go___closed__1; size_t lean_usize_of_nat(lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956_(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_isJpCases_x3f_go___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Internalize_internalizeCodeDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -93,27 +95,21 @@ static lean_object* l_Lean_Compiler_LCNF_Simp_collectJpCasesInfo___closed__3; static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJmp_x3f___closed__1; lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Internalize_internalizeFunDecl___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_RBNode_any___at_Lean_Compiler_LCNF_Simp_JpCasesInfoMap_isCandidate___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJmpArgsAtJp___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJmpArgsAtJp(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_RBNode_revFold___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__4___boxed(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Simp_withDiscrCtorImp_updateCtx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__8___closed__1; lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Simp_CtorInfo_getName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_eraseCode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -129,7 +125,6 @@ lean_object* l_Lean_Compiler_LCNF_Internalize_internalizeParam(lean_object*, lea static lean_object* l_Lean_Compiler_LCNF_Simp_collectJpCasesInfo___closed__1; extern lean_object* l_Lean_Compiler_LCNF_instInhabitedArg; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_CasesCore_getCtorNames(lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___closed__1; @@ -139,17 +134,21 @@ extern lean_object* l_Lean_inheritedTraceOptions; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_instInhabitedCasesCore(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14; lean_object* l_Lean_Compiler_LCNF_attachCodeDecls(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBTree_toList___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__3(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_extractJpCases_go(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___lambda__1___closed__2; static lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_extractJpCases_go___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Simp_collectJpCasesInfo_go___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt___closed__1; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3; extern lean_object* l_Lean_NameSet_empty; LEAN_EXPORT lean_object* l___private_Init_Data_Array_BasicAux_0__mapMonoMImp___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visit___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15; static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__6___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___spec__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,26 +159,26 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Compiler_LCN uint8_t l_Lean_NameSet_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4; lean_object* lean_panic_fn(lean_object*, lean_object*); uint8_t l___private_Lean_Compiler_LCNF_DependsOn_0__Lean_Compiler_LCNF_depOn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9; static lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___spec__8___closed__4; static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__7; lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2; extern lean_object* l_Lean_Compiler_LCNF_instInhabitedParam; static lean_object* l_panic___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_extractJpCases_go___spec__1___closed__1; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_mkJpAlt_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdSet_insert___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_JpCasesInfoMap_isCandidate___boxed(lean_object*); static lean_object* l_panic___at___private_Lean_Compiler_LCNF_Simp_JpCases_0__Lean_Compiler_LCNF_Simp_extractJpCases_go___spec__1___closed__3; lean_object* l_List_reverse___rarg(lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15; lean_object* l_Lean_mkHashMapImp___rarg(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17; uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_BasicAux_0__mapMonoMImp_go___at_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visit___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateAltCodeImp(lean_object*, lean_object*); @@ -195,17 +194,18 @@ static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f_visitJp_x3f___lamb LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_Simp_JpCasesInfoMap_isCandidate(lean_object*); lean_object* l_Lean_Compiler_LCNF_Simp_findCtor_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922_(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18; static lean_object* l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__2; lean_object* lean_array_get_size(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5; uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_isJpCases_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Simp_collectJpCasesInfo___closed__4; lean_object* l_Lean_Compiler_LCNF_mkAuxFunDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_collectJpCasesInfo_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Simp_instInhabitedJpCasesInfo; static lean_object* l_Lean_Compiler_LCNF_Simp_collectJpCasesInfo___closed__2; @@ -7861,7 +7861,7 @@ lean_dec(x_3); return x_9; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1() { _start: { lean_object* x_1; @@ -7869,27 +7869,27 @@ x_1 = lean_mk_string_from_bytes("Lean", 4); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2; x_2 = l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4() { _start: { lean_object* x_1; @@ -7897,17 +7897,17 @@ x_1 = lean_mk_string_from_bytes("LCNF", 4); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6() { _start: { lean_object* x_1; @@ -7915,17 +7915,17 @@ x_1 = lean_mk_string_from_bytes("initFn", 6); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8() { _start: { lean_object* x_1; @@ -7933,47 +7933,47 @@ x_1 = lean_mk_string_from_bytes("_@", 2); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10; x_2 = l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13() { _start: { lean_object* x_1; @@ -7981,17 +7981,17 @@ x_1 = lean_mk_string_from_bytes("Simp", 4); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15() { _start: { lean_object* x_1; @@ -7999,17 +7999,17 @@ x_1 = lean_mk_string_from_bytes("JpCases", 7); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17() { _start: { lean_object* x_1; @@ -8017,33 +8017,33 @@ x_1 = lean_mk_string_from_bytes("_hyg", 4); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18; -x_2 = lean_unsigned_to_nat(3922u); +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18; +x_2 = lean_unsigned_to_nat(3956u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__4; x_3 = 0; -x_4 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19; +x_4 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -8153,45 +8153,45 @@ l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__6 = _init_l_Lean lean_mark_persistent(l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__6); l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__7 = _init_l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__7(); lean_mark_persistent(l_Lean_Compiler_LCNF_Simp_simpJpCases_x3f___lambda__1___closed__7); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__1); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__2); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__3); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__4); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__5); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__6); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__7); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__8); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__9); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__10); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__11); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__12); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__13); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__14); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__15); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__16); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__17); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__18); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922____closed__19); -if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3922_(lean_io_mk_world()); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__1); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__2); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__3); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__4); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__5); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__6); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__7); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__8); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__9); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__10); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__11); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__12); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__13); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__14); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__15); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__16); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__17); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__18); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956____closed__19); +if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Simp_JpCases___hyg_3956_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c b/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c index 8ce714d5505d..0ef0885f9e6e 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Specialize.c @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_LetDecl_updateValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -25,12 +24,15 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_LetValue_forFVarM___at_Lean_Compil LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_shouldSpecialize___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Internalize_internalizeCode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_expandCodeDecls_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13; static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__18; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_getRemainingArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_isGround___rarg___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6; static lean_object* l_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___closed__2; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_cacheSpec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7; lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Simp_withDiscrCtorImp_updateCtx___spec__5(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__11; @@ -69,6 +71,7 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_isGround___at_Lean_Comp lean_object* l___private_Lean_Compiler_LCNF_CompilerM_0__Lean_Compiler_LCNF_updateFunDeclImp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__6; static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__5___closed__4; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14; static lean_object* l_Lean_Compiler_LCNF_specialize___closed__2; static lean_object* l_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___closed__1; lean_object* l_Lean_SMap_find_x3f___at_Lean_Compiler_getCachedSpecialization___spec__1(lean_object*, lean_object*); @@ -77,13 +80,14 @@ static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__ static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_cacheSpec___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Specialize_expandCodeDecls___spec__2(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181_(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Compiler_LCNF_FunDeclCore_toExprM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_allFVarM___at_Lean_Compiler_LCNF_Specialize_shouldSpecialize___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_mkSpecDecl_go___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -113,11 +117,11 @@ static lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl___closed__2; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_shouldSpecialize___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specCacheExt; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10; lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Decl_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_ToExpr_abstractM___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_specialize___closed__1; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Expr_forFVarM___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__5(lean_object*, lean_object*); lean_object* l___private_Lean_Compiler_LCNF_CompilerM_0__Lean_Compiler_LCNF_normArgImp(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -178,18 +182,17 @@ lean_object* l_Lean_Compiler_LCNF_Closure_collectArg(lean_object*, lean_object*, LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__8; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_findSpecCache_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_HashMapImp_contains___at_Lean_Compiler_LCNF_Specialize_Collector_collect___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15; static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__1; lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Expr_forFVarM___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__5___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__17; lean_object* l_Lean_Compiler_LCNF_Internalize_internalizeParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1; static lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl___closed__3; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15; lean_object* l_Lean_Compiler_LCNF_getDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__1___closed__2; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -199,10 +202,10 @@ lean_object* l_Lean_Compiler_LCNF_ToExpr_mkLambdaM___boxed(lean_object*, lean_ob LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_isGround(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_visitFunDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__4(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_main(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__9; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2; static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__7; lean_object* l_Lean_Compiler_LCNF_LetValue_toExpr(lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__4___closed__1; @@ -229,16 +232,16 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lam static lean_object* l_Lean_addTrace___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__5___closed__3; lean_object* lean_name_append_index_after(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_expandCodeDecls___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5; LEAN_EXPORT lean_object* l___private_Init_Data_Array_BasicAux_0__mapMonoMImp___at_Lean_Compiler_LCNF_Specialize_visitCode___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_allFVarM___at_Lean_Compiler_LCNF_Specialize_isGround___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_mkSpecDecl_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_getSpecParamInfo_x3f___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_shouldSpecialize___spec__3___closed__1; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4; static lean_object* l_Lean_Compiler_LCNF_Specialize_cacheSpec___closed__1; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7; LEAN_EXPORT lean_object* l_panic___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_getRemainingArgs___spec__1(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_allFVarM___at_Lean_Compiler_LCNF_Specialize_isGround___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____lambda__1___closed__5; lean_object* l_Lean_HashMap_insert___at_Lean_Compiler_LCNF_addFVarSubst___spec__1(lean_object*, lean_object*, lean_object*); @@ -256,8 +259,6 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_allFVarM___at_Lean_Compiler_LCNF_S LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_getRemainingArgs(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__10; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1; lean_object* l_Lean_Compiler_LCNF_Arg_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_CodeDecl_fvarId(lean_object*); @@ -269,6 +270,7 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Comp lean_object* l_Lean_Compiler_LCNF_allFVarM_go___at_Lean_Compiler_LCNF_allFVar___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Decl_specialize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__6___closed__2; +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194_(lean_object*); lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Closure_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); @@ -277,12 +279,14 @@ lean_object* l_Array_ofSubarray___rarg(lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdSet_insert___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_OptionT_instMonadOptionT___rarg(lean_object*); lean_object* lean_erase_macro_scopes(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9; lean_object* lean_expr_instantiate_rev(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Compiler_LCNF_Decl_instantiateValueLevelParams(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__5; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkHashMapImp___rarg(lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11; static lean_object* l_Lean_Compiler_LCNF_Specialize_instInhabitedCacheEntry___closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___boxed(lean_object**); lean_object* l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_updateAltCodeImp(lean_object*, lean_object*); @@ -293,7 +297,6 @@ uint8_t l_Lean_Expr_hasFVar(lean_object*); extern lean_object* l_Id_instMonadId; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_State_decls___default; lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_withParams___spec__1(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Expr_fvar___override(lean_object*); @@ -303,7 +306,6 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_getRemainingArgs___boxe LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_Specialize_Collector_collect___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Expr_forFVarM___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__5___closed__4; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9; uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1933_(lean_object*); lean_object* l_Lean_Expr_instantiateLevelParamsNoCache(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_ToExpr_withParams_go___at_Lean_Compiler_LCNF_Specialize_mkKey___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -321,23 +323,21 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_visitCode___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__2___closed__1; -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6; static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_instMonadScopeSpecializeM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__5___closed__3; lean_object* l_Lean_Compiler_LCNF_FunDeclCore_toExpr(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_allFVarM___at_Lean_Compiler_LCNF_Specialize_withLetDecl___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__13; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_getSpecParamInfo_x3f___at_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_Collector_collect___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Specialize_isGround___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Compiler_LCNF_Specialize_shouldSpecialize___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13; lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l_Lean_Compiler_LCNF_Specialize_mkSpecDecl___closed__1; static lean_object* l_Lean_Compiler_LCNF_Specialize_specializeApp_x3f___lambda__3___closed__3; @@ -10207,7 +10207,7 @@ lean_dec(x_1); return x_12; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10217,7 +10217,7 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10227,27 +10227,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5() { _start: { lean_object* x_1; @@ -10255,17 +10255,17 @@ x_1 = lean_mk_string_from_bytes("initFn", 6); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7() { _start: { lean_object* x_1; @@ -10273,57 +10273,57 @@ x_1 = lean_mk_string_from_bytes("_@", 2); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11; x_2 = l_Lean_Compiler_LCNF_Specialize_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_50____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13() { _start: { lean_object* x_1; @@ -10331,33 +10331,33 @@ x_1 = lean_mk_string_from_bytes("_hyg", 4); return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13; +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14; -x_2 = lean_unsigned_to_nat(5181u); +x_1 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14; +x_2 = lean_unsigned_to_nat(5194u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1; x_3 = 1; -x_4 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15; +x_4 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -10647,37 +10647,37 @@ l_Lean_Compiler_LCNF_specialize___closed__3 = _init_l_Lean_Compiler_LCNF_special lean_mark_persistent(l_Lean_Compiler_LCNF_specialize___closed__3); l_Lean_Compiler_LCNF_specialize = _init_l_Lean_Compiler_LCNF_specialize(); lean_mark_persistent(l_Lean_Compiler_LCNF_specialize); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__1); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__2); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__3); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__4); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__5); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__6); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__7); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__8); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__9); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__10); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__11); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__12); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__13); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__14); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181____closed__15); -if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5181_(lean_io_mk_world()); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__1); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__2); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__3); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__4); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__5); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__6); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__7); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__8); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__9); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__10); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__11); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__12); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__13); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__14); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194____closed__15); +if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_Specialize___hyg_5194_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Compiler/LCNF/Testing.c b/stage0/stdlib/Lean/Compiler/LCNF/Testing.c index 7e451245fbdb..aa5b6260b84e 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/Testing.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/Testing.c @@ -51,7 +51,6 @@ extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Testing_assertSize___spec__1(size_t, size_t, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Testing_assertSize___lambda__1___closed__3; -uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Testing_assert___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Testing_assertIsAtFixPoint___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Code_containsConst_goLetValue___boxed(lean_object*, lean_object*); @@ -113,6 +112,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Compiler_LCNF_Testing_0__Lean_Compiler LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Testing_getDecls___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Testing_assert(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Testing_TestM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_Testing_assertIsAtFixPoint___lambda__1___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Testing_SimpleAssertionM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2893,7 +2893,7 @@ else lean_object* x_10; lean_object* x_11; uint8_t x_12; x_10 = lean_array_fget(x_4, x_6); x_11 = lean_array_fget(x_5, x_6); -x_12 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5757_(x_10, x_11); +x_12 = l___private_Lean_Compiler_LCNF_Basic_0__Lean_Compiler_LCNF_beqDecl____x40_Lean_Compiler_LCNF_Basic___hyg_5796_(x_10, x_11); if (x_12 == 0) { uint8_t x_13; diff --git a/stage0/stdlib/Lean/DocString.c b/stage0/stdlib/Lean/DocString.c index 759c787fc59e..f1cbd38039b4 100644 --- a/stage0/stdlib/Lean/DocString.c +++ b/stage0/stdlib/Lean/DocString.c @@ -13,14 +13,15 @@ #ifdef __cplusplus extern "C" { #endif +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_56____closed__2; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_saveLine(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_4_(lean_object*); lean_object* l_Lean_indentD(lean_object*); static lean_object* l_Lean_addBuiltinDocString___closed__1; @@ -30,6 +31,7 @@ lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDocStringText(lean_object*); LEAN_EXPORT lean_object* l_Lean_getModuleDoc_x3f___boxed(lean_object*, lean_object*); lean_object* l_String_Iterator_next(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195_(lean_object*); LEAN_EXPORT lean_object* l_Lean_getDocStringText___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_removeLeadingSpaces(lean_object*); LEAN_EXPORT lean_object* l_Lean_findDocString_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -39,6 +41,7 @@ lean_object* lean_string_utf8_byte_size(lean_object*); lean_object* lean_string_push(lean_object*, uint32_t); uint32_t l_String_Iterator_curr(lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_findNextLine(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_findDocString_x3f___spec__1(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); @@ -51,28 +54,28 @@ lean_object* l_Lean_MessageData_ofSyntax(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_docStringExt; LEAN_EXPORT lean_object* l_Lean_addMainModuleDoc(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6; lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3; lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* lean_list_to_array(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3; lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3; +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1; LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1; static lean_object* l_Lean_getDocStringText___rarg___closed__3; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_getDocString(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_builtinDocStrings; static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_56____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5; LEAN_EXPORT lean_object* l_Lean_addDocString___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_getMainModuleDoc(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_56____closed__1; LEAN_EXPORT lean_object* l_Lean_getModuleDoc_x3f(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5; lean_object* l_Lean_throwErrorAt___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_getDocString___boxed(lean_object*); static lean_object* l_Lean_getModuleDoc_x3f___closed__1; @@ -80,17 +83,15 @@ LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_moduleDocExt; LEAN_EXPORT lean_object* l_Lean_addDocString(lean_object*); lean_object* lean_string_length(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2; +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6; static lean_object* l_Lean_addMainModuleDoc___closed__1; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033_(lean_object*); lean_object* l_Lean_Environment_getModuleIdx_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* l_Lean_mkMapDeclarationExtension___rarg(lean_object*, lean_object*); lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4; static lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1; uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); static lean_object* l_Lean_getDocStringText___rarg___closed__2; @@ -99,13 +100,12 @@ lean_object* l_Lean_instInhabitedPersistentArray(lean_object*); static lean_object* l_Lean_getMainModuleDoc___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_findDocString_x3f___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2; uint8_t l_String_Iterator_atEnd(lean_object*); LEAN_EXPORT lean_object* l_String_Iterator_find___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__1(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_getDocStringText___rarg___closed__1; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_addDocString_x27(lean_object*); LEAN_EXPORT lean_object* l_Lean_getMainModuleDoc___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_4_(lean_object* x_1) { @@ -741,7 +741,7 @@ x_6 = l_Lean_findDocString_x3f(x_1, x_2, x_5, x_4); return x_6; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -750,23 +750,23 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1; +x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3() { _start: { size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 5; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2; -x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2; +x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1; x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_2); @@ -777,15 +777,15 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3; return x_2; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1() { _start: { lean_object* x_1; @@ -793,17 +793,17 @@ x_1 = lean_mk_string_from_bytes("moduleDocExt", 12); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_56____closed__1; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3() { _start: { lean_object* x_1; @@ -812,7 +812,7 @@ lean_closure_set(x_1, 0, lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4() { _start: { lean_object* x_1; @@ -820,22 +820,22 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PersistentArray_push___rarg), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4; -x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5; -x_4 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3; +x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4; +x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5; +x_4 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3; x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -844,20 +844,20 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6; x_3 = l_Lean_registerSimplePersistentEnvExtension___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1(x_1); +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1(x_1); lean_dec(x_1); return x_2; } @@ -1141,25 +1141,25 @@ l_Lean_addBuiltinDocString___closed__1 = _init_l_Lean_addBuiltinDocString___clos lean_mark_persistent(l_Lean_addBuiltinDocString___closed__1); l_Lean_addDocString___rarg___lambda__1___closed__1 = _init_l_Lean_addDocString___rarg___lambda__1___closed__1(); lean_mark_persistent(l_Lean_addDocString___rarg___lambda__1___closed__1); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__1); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__2); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____lambda__1___closed__3); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__1); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__2); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__3); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__4); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__5); -l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2033____closed__6); -if (builtin) {res = l_Lean_initFn____x40_Lean_DocString___hyg_2033_(lean_io_mk_world()); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__1); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__2); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____lambda__1___closed__3); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__1); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__2); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__3); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__4); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__5); +l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_2195____closed__6); +if (builtin) {res = l_Lean_initFn____x40_Lean_DocString___hyg_2195_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l___private_Lean_DocString_0__Lean_moduleDocExt = lean_io_result_get_value(res); lean_mark_persistent(l___private_Lean_DocString_0__Lean_moduleDocExt); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c index 9a10e5b3e1d8..72db1b00e4fb 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c @@ -373,7 +373,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_4); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c index 15812df3660e..0676571158a0 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c @@ -4891,7 +4891,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_3); diff --git a/stage0/stdlib/Lean/Elab/Structure.c b/stage0/stdlib/Lean/Elab/Structure.c index 20b47cdeab34..caeb78cb7408 100644 --- a/stage0/stdlib/Lean/Elab/Structure.c +++ b/stage0/stdlib/Lean/Elab/Structure.c @@ -31,6 +31,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFie LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,7 +93,8 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1; static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__14; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabStructure___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -105,7 +107,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11; lean_object* l_Lean_indentD(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; @@ -158,7 +159,6 @@ lean_object* l_Lean_instBEqLocalInstance___boxed(lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkFreshId___at_Lean_Meta_mkFreshExprMVarAt___spec__2___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -208,6 +208,7 @@ lean_object* l_Lean_Elab_Term_declareTacticSyntax(lean_object*, lean_object*, le lean_object* l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); @@ -234,6 +235,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Stru LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldInfo_isSubobject___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2; @@ -287,7 +289,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_ lean_object* l_instHashableArray___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; size_t lean_ptr_addr(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__1; @@ -306,7 +307,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_ge LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_abstract(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -343,7 +344,6 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_process LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -351,7 +351,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co static lean_object* l_Lean_Elab_Command_elabStructure___closed__12; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___boxed(lean_object**); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12; static lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___closed__1; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__4; @@ -375,7 +374,6 @@ lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_obje LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__15; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerStructure(lean_object*, lean_object*); @@ -404,6 +402,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ lean_object* l_Lean_Elab_Term_applyAttributesAt(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454_(lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_4654____closed__5; @@ -472,7 +471,6 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(lean_object*, lean_object*); @@ -520,7 +518,6 @@ static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structu static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__24; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__6; lean_object* l_Lean_Syntax_getSepArgs(lean_object*); @@ -536,7 +533,6 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFiel lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_580____closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -562,7 +558,6 @@ static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0 static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__19; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__10; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -583,6 +578,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getOptDerivingClasses___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; @@ -602,7 +599,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Stru LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_mkNoConfusionEnum_mkToCtorIdx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__2___boxed(lean_object**); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -623,6 +619,7 @@ lean_object* l_Lean_Elab_Term_applyAttributesAt___boxed(lean_object*, lean_objec uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13; lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -723,7 +720,6 @@ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__L lean_object* l_Lean_Level_getLevelOffset(lean_object*); static size_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3; lean_object* l_Lean_Expr_getForallBody(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshLevelMVarsFor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -864,6 +860,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStr LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_ofNat___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14; lean_object* l_Lean_Meta_removeUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__19; static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__12; @@ -884,7 +881,6 @@ static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___cl lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_580____closed__8; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451_(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__16; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4; @@ -921,6 +917,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNew LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___lambda__1(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__2; @@ -935,6 +932,7 @@ lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Elab_Command_elabStructure___closed__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2; static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3; @@ -946,6 +944,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStr static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_345____closed__13; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6; lean_object* l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; @@ -953,7 +952,6 @@ lean_object* l_Lean_Elab_Modifiers_addAttribute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__20; lean_object* l_Array_sequenceMap___at_Lean_Elab_elabDeriving___spec__2(lean_object*, lean_object*); @@ -970,6 +968,7 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Stru static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal(lean_object*, lean_object*, lean_object*); @@ -1025,6 +1024,7 @@ lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_objec static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11; LEAN_EXPORT lean_object* l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -12291,7 +12291,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_c lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2; -x_3 = lean_unsigned_to_nat(451u); +x_3 = lean_unsigned_to_nat(452u); x_4 = lean_unsigned_to_nat(68u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -12522,78 +12522,137 @@ x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Elab_Structure_0__L return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { _start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; +lean_object* x_21; lean_object* x_22; +lean_inc(x_13); lean_inc(x_2); -lean_inc(x_1); -x_22 = l_Lean_Name_append(x_1, x_2); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_3, x_19, x_20, x_21); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_unbox(x_24); -lean_dec(x_24); -lean_inc(x_20); +x_21 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_1, x_2, x_13); lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); -lean_inc(x_15); -x_27 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_26, x_22, x_15, x_16, x_17, x_18, x_19, x_20, x_25); -if (lean_obj_tag(x_27) == 0) +lean_inc(x_14); +lean_inc(x_2); +lean_inc(x_4); +lean_inc(x_3); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_21, x_3, x_4, x_2, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_22) == 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; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_28 = lean_ctor_get(x_27, 0); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +lean_inc(x_2); +lean_inc(x_5); +x_25 = l_Lean_Name_append(x_5, x_2); +x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_6, x_18, x_19, x_24); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); +lean_dec(x_26); +x_29 = lean_unbox(x_27); lean_dec(x_27); -x_30 = lean_st_ref_get(x_20, x_29); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_30 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_29, x_25, x_14, x_15, x_16, x_17, x_18, x_19, x_28); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; x_31 = lean_ctor_get(x_30, 0); lean_inc(x_31); x_32 = lean_ctor_get(x_30, 1); lean_inc(x_32); lean_dec(x_30); -x_33 = lean_ctor_get(x_31, 0); -lean_inc(x_33); -lean_dec(x_31); -x_34 = 1; -x_35 = l_Lean_findDocString_x3f(x_33, x_4, x_34, x_32); -x_36 = lean_ctor_get(x_35, 0); +x_33 = lean_st_ref_get(x_19, x_32); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_ctor_get(x_34, 0); lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -lean_inc(x_28); -x_38 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_28, x_36, x_15, x_16, x_17, x_18, x_19, x_20, x_37); -x_39 = lean_ctor_get(x_38, 1); +lean_dec(x_34); +x_37 = 1; +x_38 = l_Lean_findDocString_x3f(x_36, x_7, x_37, x_35); +x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); lean_dec(x_38); -x_40 = 1; -lean_inc(x_14); -lean_inc(x_2); -x_41 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_41, 0, x_2); -lean_ctor_set(x_41, 1, x_28); -lean_ctor_set(x_41, 2, x_14); -lean_ctor_set(x_41, 3, x_5); -lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_40); -x_42 = lean_array_push(x_6, x_41); -x_43 = lean_unsigned_to_nat(1u); -x_44 = lean_nat_add(x_7, x_43); -lean_dec(x_7); -x_45 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_8, x_2, x_14); -x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_1, x_9, x_10, x_11, x_12, x_44, x_42, x_45, x_13, x_15, x_16, x_17, x_18, x_19, x_20, x_39); -return x_46; +lean_inc(x_31); +x_41 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_31, x_39, x_14, x_15, x_16, x_17, x_18, x_19, x_40); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = 1; +x_44 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_44, 0, x_2); +lean_ctor_set(x_44, 1, x_31); +lean_ctor_set(x_44, 2, x_13); +lean_ctor_set(x_44, 3, x_23); +lean_ctor_set_uint8(x_44, sizeof(void*)*4, x_43); +x_45 = lean_array_push(x_8, x_44); +x_46 = lean_unsigned_to_nat(1u); +x_47 = lean_nat_add(x_9, x_46); +lean_dec(x_9); +x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_10, x_11, x_4, x_12, x_47, x_45, x_21, x_3, x_14, x_15, x_16, x_17, x_18, x_19, x_42); +return x_48; } else { -uint8_t x_47; -lean_dec(x_20); +uint8_t x_49; +lean_dec(x_23); +lean_dec(x_21); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_49 = !lean_is_exclusive(x_30); +if (x_49 == 0) +{ +return x_30; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_30, 0); +x_51 = lean_ctor_get(x_30, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_30); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +uint8_t x_53; +lean_dec(x_21); lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); @@ -12610,25 +12669,25 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_47 = !lean_is_exclusive(x_27); -if (x_47 == 0) +x_53 = !lean_is_exclusive(x_22); +if (x_53 == 0) { -return x_27; +return x_22; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_27, 0); -x_49 = lean_ctor_get(x_27, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_27); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_22, 0); +x_55 = lean_ctor_get(x_22, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_22); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } } @@ -12962,177 +13021,117 @@ x_40 = lean_ctor_get(x_39, 2); lean_inc(x_40); if (lean_obj_tag(x_40) == 0) { -lean_object* x_41; uint8_t x_42; lean_object* x_43; +lean_object* x_41; uint8_t x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); x_42 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_27); -lean_inc(x_4); -lean_inc(x_9); -x_43 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_8, x_9, x_4, x_27, x_10, x_11, x_12, x_13, x_14, x_15, x_34); -if (lean_obj_tag(x_43) == 0) -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; lean_object* x_48; -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); -lean_inc(x_45); -lean_dec(x_43); lean_inc(x_27); -x_46 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1___boxed), 21, 13); -lean_closure_set(x_46, 0, x_1); -lean_closure_set(x_46, 1, x_27); -lean_closure_set(x_46, 2, x_39); -lean_closure_set(x_46, 3, x_41); -lean_closure_set(x_46, 4, x_44); -lean_closure_set(x_46, 5, x_7); -lean_closure_set(x_46, 6, x_6); -lean_closure_set(x_46, 7, x_8); -lean_closure_set(x_46, 8, x_2); -lean_closure_set(x_46, 9, x_3); -lean_closure_set(x_46, 10, x_4); -lean_closure_set(x_46, 11, x_5); -lean_closure_set(x_46, 12, x_9); -x_47 = 0; -x_48 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_27, x_42, x_29, x_46, x_47, x_10, x_11, x_12, x_13, x_14, x_15, x_45); -return x_48; +x_43 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1___boxed), 20, 12); +lean_closure_set(x_43, 0, x_8); +lean_closure_set(x_43, 1, x_27); +lean_closure_set(x_43, 2, x_9); +lean_closure_set(x_43, 3, x_4); +lean_closure_set(x_43, 4, x_1); +lean_closure_set(x_43, 5, x_39); +lean_closure_set(x_43, 6, x_41); +lean_closure_set(x_43, 7, x_7); +lean_closure_set(x_43, 8, x_6); +lean_closure_set(x_43, 9, x_2); +lean_closure_set(x_43, 10, x_3); +lean_closure_set(x_43, 11, x_5); +x_44 = 0; +x_45 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_27, x_42, x_29, x_43, x_44, x_10, x_11, x_12, x_13, x_14, x_15, x_34); +return x_45; } else { -uint8_t x_49; -lean_dec(x_41); +lean_object* x_46; uint8_t x_47; lean_object* x_48; +lean_dec(x_40); +x_46 = lean_ctor_get(x_39, 0); +lean_inc(x_46); +x_47 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); lean_dec(x_39); -lean_dec(x_29); -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_43); -if (x_49 == 0) -{ -return x_43; -} -else +lean_inc(x_29); +x_48 = l_Lean_Meta_getStructureName(x_29, x_12, x_13, x_14, x_15, x_34); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_43, 0); -x_51 = lean_ctor_get(x_43, 1); -lean_inc(x_51); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); lean_inc(x_50); -lean_dec(x_43); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} -} -} -else +lean_dec(x_48); +lean_inc(x_49); +x_51 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_7, x_49, x_14, x_15, x_50); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +if (lean_obj_tag(x_52) == 0) { -lean_object* x_53; uint8_t x_54; lean_object* x_55; -lean_dec(x_40); -x_53 = lean_ctor_get(x_39, 0); +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; +lean_dec(x_27); +x_53 = lean_ctor_get(x_51, 1); lean_inc(x_53); -x_54 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); -lean_dec(x_39); -lean_inc(x_29); -x_55 = l_Lean_Meta_getStructureName(x_29, x_12, x_13, x_14, x_15, x_34); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_56 = lean_ctor_get(x_55, 0); +lean_dec(x_51); +x_54 = lean_st_ref_get(x_15, x_53); +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); +lean_dec(x_54); +x_57 = lean_ctor_get(x_55, 0); lean_inc(x_57); lean_dec(x_55); -lean_inc(x_56); -x_58 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_7, x_56, x_14, x_15, x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -if (lean_obj_tag(x_59) == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; -lean_dec(x_27); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = lean_st_ref_get(x_15, x_60); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_ctor_get(x_62, 0); -lean_inc(x_64); -lean_dec(x_62); -x_65 = 1; -lean_inc(x_56); -x_66 = l_Lean_getStructureFieldsFlattened(x_64, x_56, x_65); -lean_inc(x_53); -x_67 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3___boxed), 20, 12); -lean_closure_set(x_67, 0, x_1); -lean_closure_set(x_67, 1, x_53); -lean_closure_set(x_67, 2, x_7); -lean_closure_set(x_67, 3, x_6); -lean_closure_set(x_67, 4, x_8); -lean_closure_set(x_67, 5, x_2); -lean_closure_set(x_67, 6, x_3); -lean_closure_set(x_67, 7, x_4); -lean_closure_set(x_67, 8, x_5); -lean_closure_set(x_67, 9, x_9); -lean_closure_set(x_67, 10, x_56); -lean_closure_set(x_67, 11, x_66); -x_68 = 0; -x_69 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_53, x_54, x_29, x_67, x_68, x_10, x_11, x_12, x_13, x_14, x_15, x_63); -return x_69; +x_58 = 1; +lean_inc(x_49); +x_59 = l_Lean_getStructureFieldsFlattened(x_57, x_49, x_58); +lean_inc(x_46); +x_60 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3___boxed), 20, 12); +lean_closure_set(x_60, 0, x_1); +lean_closure_set(x_60, 1, x_46); +lean_closure_set(x_60, 2, x_7); +lean_closure_set(x_60, 3, x_6); +lean_closure_set(x_60, 4, x_8); +lean_closure_set(x_60, 5, x_2); +lean_closure_set(x_60, 6, x_3); +lean_closure_set(x_60, 7, x_4); +lean_closure_set(x_60, 8, x_5); +lean_closure_set(x_60, 9, x_9); +lean_closure_set(x_60, 10, x_49); +lean_closure_set(x_60, 11, x_59); +x_61 = 0; +x_62 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_46, x_47, x_29, x_60, x_61, x_10, x_11, x_12, x_13, x_14, x_15, x_56); +return x_62; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -lean_dec(x_59); -lean_dec(x_53); -x_70 = lean_ctor_get(x_58, 1); -lean_inc(x_70); -lean_dec(x_58); -x_71 = lean_box(0); -x_72 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_9, x_56, x_71); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_52); +lean_dec(x_46); +x_63 = lean_ctor_get(x_51, 1); +lean_inc(x_63); +lean_dec(x_51); +x_64 = lean_box(0); +x_65 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_9, x_49, x_64); lean_inc(x_1); lean_inc(x_29); -x_73 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed), 19, 9); -lean_closure_set(x_73, 0, x_29); -lean_closure_set(x_73, 1, x_6); -lean_closure_set(x_73, 2, x_8); -lean_closure_set(x_73, 3, x_27); -lean_closure_set(x_73, 4, x_1); -lean_closure_set(x_73, 5, x_2); -lean_closure_set(x_73, 6, x_3); -lean_closure_set(x_73, 7, x_4); -lean_closure_set(x_73, 8, x_5); -x_74 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_7, x_72, x_29, x_73, x_10, x_11, x_12, x_13, x_14, x_15, x_70); -return x_74; +x_66 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed), 19, 9); +lean_closure_set(x_66, 0, x_29); +lean_closure_set(x_66, 1, x_6); +lean_closure_set(x_66, 2, x_8); +lean_closure_set(x_66, 3, x_27); +lean_closure_set(x_66, 4, x_1); +lean_closure_set(x_66, 5, x_2); +lean_closure_set(x_66, 6, x_3); +lean_closure_set(x_66, 7, x_4); +lean_closure_set(x_66, 8, x_5); +x_67 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_7, x_65, x_29, x_66, x_10, x_11, x_12, x_13, x_14, x_15, x_63); +return x_67; } } else { -uint8_t x_75; -lean_dec(x_53); +uint8_t x_68; +lean_dec(x_46); lean_dec(x_29); lean_dec(x_27); lean_dec(x_15); @@ -13150,23 +13149,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_55); -if (x_75 == 0) +x_68 = !lean_is_exclusive(x_48); +if (x_68 == 0) { -return x_55; +return x_48; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_55, 0); -x_77 = lean_ctor_get(x_55, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_55); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_48, 0); +x_70 = lean_ctor_get(x_48, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_48); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; } } } @@ -13174,45 +13173,45 @@ return x_78; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_31, 0); -lean_inc(x_79); +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_31, 0); +lean_inc(x_72); lean_dec(x_31); -x_80 = lean_ctor_get(x_79, 2); -lean_inc(x_80); -lean_dec(x_79); +x_73 = lean_ctor_get(x_72, 2); +lean_inc(x_73); +lean_dec(x_72); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_80); -x_81 = lean_infer_type(x_80, x_12, x_13, x_14, x_15, x_30); -if (lean_obj_tag(x_81) == 0) +lean_inc(x_73); +x_74 = lean_infer_type(x_73, x_12, x_13, x_14, x_15, x_30); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_82); +lean_inc(x_75); lean_inc(x_29); -x_84 = l_Lean_Meta_isExprDefEq(x_29, x_82, x_12, x_13, x_14, x_15, x_83); -if (lean_obj_tag(x_84) == 0) +x_77 = l_Lean_Meta_isExprDefEq(x_29, x_75, x_12, x_13, x_14, x_15, x_76); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_85; uint8_t x_86; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_unbox(x_85); -lean_dec(x_85); -if (x_86 == 0) +lean_object* x_78; uint8_t x_79; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_unbox(x_78); +lean_dec(x_78); +if (x_79 == 0) { -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; uint8_t x_104; -lean_dec(x_80); +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; uint8_t x_97; +lean_dec(x_73); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -13221,86 +13220,86 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_87 = lean_ctor_get(x_84, 1); -lean_inc(x_87); -lean_dec(x_84); +x_80 = lean_ctor_get(x_77, 1); +lean_inc(x_80); +lean_dec(x_77); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_88 = l_Lean_Meta_mkHasTypeButIsExpectedMsg(x_29, x_82, x_12, x_13, x_14, x_15, x_87); -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); -lean_inc(x_90); -lean_dec(x_88); -x_91 = l_Lean_MessageData_ofName(x_27); -x_92 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; +x_81 = l_Lean_Meta_mkHasTypeButIsExpectedMsg(x_29, x_75, x_12, x_13, x_14, x_15, x_80); +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +lean_dec(x_81); +x_84 = l_Lean_MessageData_ofName(x_27); +x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; +x_86 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_84); +x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Lean_MessageData_ofName(x_4); +x_90 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_91 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8; +x_92 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); x_93 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_91); -x_94 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; +lean_ctor_set(x_93, 1, x_82); +x_94 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; x_95 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_95, 0, x_93); lean_ctor_set(x_95, 1, x_94); -x_96 = l_Lean_MessageData_ofName(x_4); -x_97 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -x_98 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8; -x_99 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -x_100 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_100, 0, x_99); -lean_ctor_set(x_100, 1, x_89); -x_101 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_102 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_102, 0, x_100); -lean_ctor_set(x_102, 1, x_101); -x_103 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_102, x_10, x_11, x_12, x_13, x_14, x_15, x_90); +x_96 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_95, x_10, x_11, x_12, x_13, x_14, x_15, x_83); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -x_104 = !lean_is_exclusive(x_103); -if (x_104 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -return x_103; +return x_96; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_103, 0); -x_106 = lean_ctor_get(x_103, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_103); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_96, 0); +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -lean_dec(x_82); +lean_object* x_101; lean_object* x_102; lean_object* x_103; +lean_dec(x_75); lean_dec(x_29); -x_108 = lean_ctor_get(x_84, 1); -lean_inc(x_108); -lean_dec(x_84); -x_109 = lean_box(0); -x_110 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_6, x_8, x_27, x_80, x_1, x_2, x_3, x_4, x_5, x_7, x_9, x_109, x_10, x_11, x_12, x_13, x_14, x_15, x_108); -return x_110; +x_101 = lean_ctor_get(x_77, 1); +lean_inc(x_101); +lean_dec(x_77); +x_102 = lean_box(0); +x_103 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_6, x_8, x_27, x_73, x_1, x_2, x_3, x_4, x_5, x_7, x_9, x_102, x_10, x_11, x_12, x_13, x_14, x_15, x_101); +return x_103; } } else { -uint8_t x_111; -lean_dec(x_82); -lean_dec(x_80); +uint8_t x_104; +lean_dec(x_75); +lean_dec(x_73); lean_dec(x_29); lean_dec(x_27); lean_dec(x_15); @@ -13318,30 +13317,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_111 = !lean_is_exclusive(x_84); -if (x_111 == 0) +x_104 = !lean_is_exclusive(x_77); +if (x_104 == 0) { -return x_84; +return x_77; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_112 = lean_ctor_get(x_84, 0); -x_113 = lean_ctor_get(x_84, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_84); -x_114 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_114, 0, x_112); -lean_ctor_set(x_114, 1, x_113); -return x_114; +lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_105 = lean_ctor_get(x_77, 0); +x_106 = lean_ctor_get(x_77, 1); +lean_inc(x_106); +lean_inc(x_105); +lean_dec(x_77); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_105); +lean_ctor_set(x_107, 1, x_106); +return x_107; } } } else { -uint8_t x_115; -lean_dec(x_80); +uint8_t x_108; +lean_dec(x_73); lean_dec(x_29); lean_dec(x_27); lean_dec(x_15); @@ -13359,30 +13358,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_115 = !lean_is_exclusive(x_81); -if (x_115 == 0) +x_108 = !lean_is_exclusive(x_74); +if (x_108 == 0) { -return x_81; +return x_74; } else { -lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_116 = lean_ctor_get(x_81, 0); -x_117 = lean_ctor_get(x_81, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_81); -x_118 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_118, 0, x_116); -lean_ctor_set(x_118, 1, x_117); -return x_118; +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_74, 0); +x_110 = lean_ctor_get(x_74, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_74); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +return x_111; } } } } else { -uint8_t x_119; +uint8_t x_112; lean_dec(x_27); lean_dec(x_15); lean_dec(x_14); @@ -13399,23 +13398,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_119 = !lean_is_exclusive(x_28); -if (x_119 == 0) +x_112 = !lean_is_exclusive(x_28); +if (x_112 == 0) { return x_28; } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_120 = lean_ctor_get(x_28, 0); -x_121 = lean_ctor_get(x_28, 1); -lean_inc(x_121); -lean_inc(x_120); +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_28, 0); +x_114 = lean_ctor_get(x_28, 1); +lean_inc(x_114); +lean_inc(x_113); lean_dec(x_28); -x_122 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_122, 0, x_120); -lean_ctor_set(x_122, 1, x_121); -return x_122; +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +return x_115; } } } @@ -13450,12 +13449,11 @@ lean_object* x_17 = _args[16]; lean_object* x_18 = _args[17]; lean_object* x_19 = _args[18]; lean_object* x_20 = _args[19]; -lean_object* x_21 = _args[20]; _start: { -lean_object* x_22; -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21); -return x_22; +lean_object* x_21; +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +return x_21; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed(lean_object** _args) { @@ -21836,7 +21834,7 @@ static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Str lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(716u); +x_3 = lean_unsigned_to_nat(717u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -21857,7 +21855,7 @@ static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Str lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(715u); +x_3 = lean_unsigned_to_nat(716u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -23639,7 +23637,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_s lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_setSourceInstImplicit___closed__1; -x_3 = lean_unsigned_to_nat(753u); +x_3 = lean_unsigned_to_nat(754u); x_4 = lean_unsigned_to_nat(9u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -24031,7 +24029,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Stru lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(777u); +x_3 = lean_unsigned_to_nat(778u); x_4 = lean_unsigned_to_nat(79u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -24340,7 +24338,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_m lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(768u); +x_3 = lean_unsigned_to_nat(769u); x_4 = lean_unsigned_to_nat(70u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -24994,7 +24992,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_m lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1; -x_3 = lean_unsigned_to_nat(760u); +x_3 = lean_unsigned_to_nat(761u); x_4 = lean_unsigned_to_nat(65u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -30583,7 +30581,7 @@ lean_dec(x_8); return x_15; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -30593,27 +30591,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1; x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_4654____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2; x_2 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4() { _start: { lean_object* x_1; @@ -30621,17 +30619,17 @@ x_1 = lean_mk_string_from_bytes("initFn", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6() { _start: { lean_object* x_1; @@ -30639,37 +30637,37 @@ x_1 = lean_mk_string_from_bytes("_@", 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7; x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8; x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_4654____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10() { _start: { lean_object* x_1; @@ -30677,17 +30675,17 @@ x_1 = lean_mk_string_from_bytes("Structure", 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12() { _start: { lean_object* x_1; @@ -30695,33 +30693,33 @@ x_1 = lean_mk_string_from_bytes("_hyg", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13; -x_2 = lean_unsigned_to_nat(16451u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13; +x_2 = lean_unsigned_to_nat(16454u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -31446,35 +31444,35 @@ l_Lean_Elab_Command_elabStructure___closed__11 = _init_l_Lean_Elab_Command_elabS lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__11); l_Lean_Elab_Command_elabStructure___closed__12 = _init_l_Lean_Elab_Command_elabStructure___closed__12(); lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__13); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451____closed__14); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16451_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__13); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454____closed__14); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_16454_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c index e9b293d7ca5c..521d08dafc56 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c @@ -15593,77 +15593,101 @@ lean_inc(x_1); x_10 = l_Lean_Elab_Tactic_getMainGoal(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_10, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_11 = lean_ctor_get(x_5, 0); lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +x_12 = lean_ctor_get(x_10, 0); lean_inc(x_12); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); lean_dec(x_10); +x_14 = lean_ctor_get(x_5, 1); +lean_inc(x_14); +x_15 = lean_ctor_get(x_5, 2); +lean_inc(x_15); +x_16 = lean_ctor_get(x_5, 3); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 4); +lean_inc(x_17); +x_18 = lean_ctor_get(x_5, 5); +lean_inc(x_18); +x_19 = !lean_is_exclusive(x_11); +if (x_19 == 0) +{ +uint8_t x_20; lean_object* x_21; lean_object* x_22; +x_20 = 1; +lean_ctor_set_uint8(x_11, 7, x_20); +x_21 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_21, 0, x_11); +lean_ctor_set(x_21, 1, x_14); +lean_ctor_set(x_21, 2, x_15); +lean_ctor_set(x_21, 3, x_16); +lean_ctor_set(x_21, 4, x_17); +lean_ctor_set(x_21, 5, x_18); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_13 = l_Lean_MVarId_assumption(x_11, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) +x_22 = l_Lean_MVarId_assumption(x_12, x_21, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_box(0); -x_16 = l_Lean_Elab_Tactic_replaceMainGoal(x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_14); -if (lean_obj_tag(x_16) == 0) +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_box(0); +x_25 = l_Lean_Elab_Tactic_replaceMainGoal(x_24, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_23); +if (lean_obj_tag(x_25) == 0) { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_16, 0); -lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_16, 0, x_19); -return x_16; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +x_28 = lean_box(0); +lean_ctor_set(x_25, 0, x_28); +return x_25; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_16, 1); -lean_inc(x_20); -lean_dec(x_16); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_25, 1); +lean_inc(x_29); +lean_dec(x_25); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; } } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_16); -if (x_23 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_25); +if (x_32 == 0) { -return x_16; +return x_25; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_16, 0); -x_25 = lean_ctor_get(x_16, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_16); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_25, 0); +x_34 = lean_ctor_get(x_25, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_25); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -uint8_t x_27; +uint8_t x_36; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -15672,29 +15696,125 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_27 = !lean_is_exclusive(x_13); -if (x_27 == 0) +x_36 = !lean_is_exclusive(x_22); +if (x_36 == 0) { -return x_13; +return x_22; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_13, 0); -x_29 = lean_ctor_get(x_13, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_13); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_22, 0); +x_38 = lean_ctor_get(x_22, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_22); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -uint8_t x_31; +uint8_t x_40; uint8_t x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; uint8_t x_47; uint8_t x_48; uint8_t x_49; uint8_t x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_40 = lean_ctor_get_uint8(x_11, 0); +x_41 = lean_ctor_get_uint8(x_11, 1); +x_42 = lean_ctor_get_uint8(x_11, 2); +x_43 = lean_ctor_get_uint8(x_11, 3); +x_44 = lean_ctor_get_uint8(x_11, 4); +x_45 = lean_ctor_get_uint8(x_11, 5); +x_46 = lean_ctor_get_uint8(x_11, 6); +x_47 = lean_ctor_get_uint8(x_11, 8); +x_48 = lean_ctor_get_uint8(x_11, 9); +x_49 = lean_ctor_get_uint8(x_11, 10); +x_50 = lean_ctor_get_uint8(x_11, 11); +lean_dec(x_11); +x_51 = 1; +x_52 = lean_alloc_ctor(0, 0, 12); +lean_ctor_set_uint8(x_52, 0, x_40); +lean_ctor_set_uint8(x_52, 1, x_41); +lean_ctor_set_uint8(x_52, 2, x_42); +lean_ctor_set_uint8(x_52, 3, x_43); +lean_ctor_set_uint8(x_52, 4, x_44); +lean_ctor_set_uint8(x_52, 5, x_45); +lean_ctor_set_uint8(x_52, 6, x_46); +lean_ctor_set_uint8(x_52, 7, x_51); +lean_ctor_set_uint8(x_52, 8, x_47); +lean_ctor_set_uint8(x_52, 9, x_48); +lean_ctor_set_uint8(x_52, 10, x_49); +lean_ctor_set_uint8(x_52, 11, x_50); +x_53 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_14); +lean_ctor_set(x_53, 2, x_15); +lean_ctor_set(x_53, 3, x_16); +lean_ctor_set(x_53, 4, x_17); +lean_ctor_set(x_53, 5, x_18); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_54 = l_Lean_MVarId_assumption(x_12, x_53, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_56 = lean_box(0); +x_57 = l_Lean_Elab_Tactic_replaceMainGoal(x_56, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_55); +if (lean_obj_tag(x_57) == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_59 = x_57; +} else { + lean_dec_ref(x_57); + x_59 = lean_box(0); +} +x_60 = lean_box(0); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); +} else { + x_61 = x_59; +} +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_62 = lean_ctor_get(x_57, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_57, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_64 = x_57; +} else { + lean_dec_ref(x_57); + x_64 = lean_box(0); +} +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(1, 2, 0); +} else { + x_65 = x_64; +} +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_63); +return x_65; +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -15703,23 +15823,57 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_31 = !lean_is_exclusive(x_10); -if (x_31 == 0) +x_66 = lean_ctor_get(x_54, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_54, 1); +lean_inc(x_67); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_68 = x_54; +} else { + lean_dec_ref(x_54); + x_68 = lean_box(0); +} +if (lean_is_scalar(x_68)) { + x_69 = lean_alloc_ctor(1, 2, 0); +} else { + x_69 = x_68; +} +lean_ctor_set(x_69, 0, x_66); +lean_ctor_set(x_69, 1, x_67); +return x_69; +} +} +} +else +{ +uint8_t x_70; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_10); +if (x_70 == 0) { return x_10; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_10, 0); -x_33 = lean_ctor_get(x_10, 1); -lean_inc(x_33); -lean_inc(x_32); +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_10, 0); +x_72 = lean_ctor_get(x_10, 1); +lean_inc(x_72); +lean_inc(x_71); lean_dec(x_10); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; } } } @@ -15834,8 +15988,8 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalAssumption_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(235u); -x_2 = lean_unsigned_to_nat(60u); +x_1 = lean_unsigned_to_nat(238u); +x_2 = lean_unsigned_to_nat(90u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -15849,7 +16003,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Elab_Tactic_evalAssumption_declRange___closed__1; x_2 = lean_unsigned_to_nat(48u); x_3 = l___regBuiltin_Lean_Elab_Tactic_evalAssumption_declRange___closed__2; -x_4 = lean_unsigned_to_nat(60u); +x_4 = lean_unsigned_to_nat(90u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -16180,7 +16334,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalContradiction_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(237u); +x_1 = lean_unsigned_to_nat(240u); x_2 = lean_unsigned_to_nat(51u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16192,7 +16346,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalContradiction_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(238u); +x_1 = lean_unsigned_to_nat(241u); x_2 = lean_unsigned_to_nat(63u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16220,7 +16374,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalContradiction_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(237u); +x_1 = lean_unsigned_to_nat(240u); x_2 = lean_unsigned_to_nat(55u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16232,7 +16386,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalContradiction_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(237u); +x_1 = lean_unsigned_to_nat(240u); x_2 = lean_unsigned_to_nat(72u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16522,7 +16676,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(240u); +x_1 = lean_unsigned_to_nat(243u); x_2 = lean_unsigned_to_nat(42u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16534,7 +16688,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(241u); +x_1 = lean_unsigned_to_nat(244u); x_2 = lean_unsigned_to_nat(54u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16562,7 +16716,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(240u); +x_1 = lean_unsigned_to_nat(243u); x_2 = lean_unsigned_to_nat(46u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -16574,7 +16728,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(240u); +x_1 = lean_unsigned_to_nat(243u); x_2 = lean_unsigned_to_nat(54u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18454,7 +18608,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntro_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(243u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18466,7 +18620,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntro_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(269u); +x_1 = lean_unsigned_to_nat(272u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18494,7 +18648,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntro_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(243u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18506,7 +18660,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntro_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(243u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(56u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18763,7 +18917,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(271u); +x_1 = lean_unsigned_to_nat(274u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18775,7 +18929,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(274u); +x_1 = lean_unsigned_to_nat(277u); x_2 = lean_unsigned_to_nat(52u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18803,7 +18957,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(271u); +x_1 = lean_unsigned_to_nat(274u); x_2 = lean_unsigned_to_nat(52u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -18815,7 +18969,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(271u); +x_1 = lean_unsigned_to_nat(274u); x_2 = lean_unsigned_to_nat(66u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -19680,7 +19834,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntros_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(276u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(27u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -19692,7 +19846,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntros_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(288u); +x_1 = lean_unsigned_to_nat(291u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -19720,7 +19874,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntros_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(276u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -19732,7 +19886,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalIntros_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(276u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(41u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20027,7 +20181,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRevert_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(290u); +x_1 = lean_unsigned_to_nat(293u); x_2 = lean_unsigned_to_nat(44u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20039,7 +20193,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRevert_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(295u); +x_1 = lean_unsigned_to_nat(298u); x_2 = lean_unsigned_to_nat(51u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20067,7 +20221,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRevert_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(290u); +x_1 = lean_unsigned_to_nat(293u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20079,7 +20233,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRevert_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(290u); +x_1 = lean_unsigned_to_nat(293u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20579,7 +20733,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(297u); +x_1 = lean_unsigned_to_nat(300u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20591,7 +20745,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(306u); +x_1 = lean_unsigned_to_nat(309u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20619,7 +20773,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(297u); +x_1 = lean_unsigned_to_nat(300u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20631,7 +20785,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(297u); +x_1 = lean_unsigned_to_nat(300u); x_2 = lean_unsigned_to_nat(56u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21109,7 +21263,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(315u); +x_1 = lean_unsigned_to_nat(318u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21121,7 +21275,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(318u); +x_1 = lean_unsigned_to_nat(321u); x_2 = lean_unsigned_to_nat(51u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21149,7 +21303,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(315u); +x_1 = lean_unsigned_to_nat(318u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21161,7 +21315,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(315u); +x_1 = lean_unsigned_to_nat(318u); x_2 = lean_unsigned_to_nat(56u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21456,7 +21610,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubstVars_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(320u); +x_1 = lean_unsigned_to_nat(323u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21468,7 +21622,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubstVars_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(321u); +x_1 = lean_unsigned_to_nat(324u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21496,7 +21650,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubstVars_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(320u); +x_1 = lean_unsigned_to_nat(323u); x_2 = lean_unsigned_to_nat(51u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21508,7 +21662,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSubstVars_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(320u); +x_1 = lean_unsigned_to_nat(323u); x_2 = lean_unsigned_to_nat(64u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -28418,7 +28572,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(406u); +x_1 = lean_unsigned_to_nat(409u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -28430,7 +28584,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(416u); +x_1 = lean_unsigned_to_nat(419u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -28458,7 +28612,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(406u); +x_1 = lean_unsigned_to_nat(409u); x_2 = lean_unsigned_to_nat(29u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -28470,7 +28624,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(406u); +x_1 = lean_unsigned_to_nat(409u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -29964,7 +30118,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(418u); +x_1 = lean_unsigned_to_nat(421u); x_2 = lean_unsigned_to_nat(26u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -29976,7 +30130,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(433u); +x_1 = lean_unsigned_to_nat(436u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30004,7 +30158,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(418u); +x_1 = lean_unsigned_to_nat(421u); x_2 = lean_unsigned_to_nat(30u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30016,7 +30170,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(418u); +x_1 = lean_unsigned_to_nat(421u); x_2 = lean_unsigned_to_nat(39u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30262,7 +30416,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRenameInaccessible _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(435u); +x_1 = lean_unsigned_to_nat(438u); x_2 = lean_unsigned_to_nat(28u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30274,7 +30428,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRenameInaccessible _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(437u); +x_1 = lean_unsigned_to_nat(440u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30302,7 +30456,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRenameInaccessible _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(435u); +x_1 = lean_unsigned_to_nat(438u); x_2 = lean_unsigned_to_nat(32u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30314,7 +30468,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRenameInaccessible _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(435u); +x_1 = lean_unsigned_to_nat(438u); x_2 = lean_unsigned_to_nat(55u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30713,7 +30867,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFirst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(439u); +x_1 = lean_unsigned_to_nat(442u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30725,7 +30879,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFirst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(448u); +x_1 = lean_unsigned_to_nat(451u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30753,7 +30907,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFirst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(439u); +x_1 = lean_unsigned_to_nat(442u); x_2 = lean_unsigned_to_nat(38u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -30765,7 +30919,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFirst_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(439u); +x_1 = lean_unsigned_to_nat(442u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31068,7 +31222,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(450u); +x_1 = lean_unsigned_to_nat(453u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31080,7 +31234,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(456u); +x_1 = lean_unsigned_to_nat(459u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31108,7 +31262,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(450u); +x_1 = lean_unsigned_to_nat(453u); x_2 = lean_unsigned_to_nat(29u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31120,7 +31274,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(450u); +x_1 = lean_unsigned_to_nat(453u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31310,7 +31464,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDbgTrace_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(458u); +x_1 = lean_unsigned_to_nat(461u); x_2 = lean_unsigned_to_nat(41u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31322,7 +31476,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDbgTrace_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(461u); +x_1 = lean_unsigned_to_nat(464u); x_2 = lean_unsigned_to_nat(29u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31350,7 +31504,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDbgTrace_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(458u); +x_1 = lean_unsigned_to_nat(461u); x_2 = lean_unsigned_to_nat(45u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31362,7 +31516,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDbgTrace_declRange _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(458u); +x_1 = lean_unsigned_to_nat(461u); x_2 = lean_unsigned_to_nat(57u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31533,7 +31687,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(463u); +x_1 = lean_unsigned_to_nat(466u); x_2 = lean_unsigned_to_nat(24u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31545,7 +31699,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(466u); +x_1 = lean_unsigned_to_nat(469u); x_2 = lean_unsigned_to_nat(35u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31573,7 +31727,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(463u); +x_1 = lean_unsigned_to_nat(466u); x_2 = lean_unsigned_to_nat(28u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -31585,7 +31739,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(463u); +x_1 = lean_unsigned_to_nat(466u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c b/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c index 27dea1a8ac5b..545c69037735 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c @@ -20,16 +20,22 @@ lean_object* l___private_Init_Util_0__outOfBounds___rarg(lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_withRWRulesSeq___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withRWRulesSeq(lean_object*, 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_throwTacticEx___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq_go___closed__1; lean_object* l_Lean_MVarId_rewrite(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabRewriteConfig___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2; +static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1; static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__3; static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__5; +static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Tactic_getFVarId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq_go___closed__4; lean_object* l_List_mapTR_loop___at_Lean_resolveGlobalConstNoOverload___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -37,7 +43,6 @@ LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_withR static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq___closed__4; lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabRewriteConfig___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_expandOptLocation(lean_object*); static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__3; @@ -60,20 +65,17 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabRewrit lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__1; lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange(lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteTarget___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__5; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_withRWRulesSeq___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); lean_object* l_List_filterMap___at_Lean_resolveGlobalConst___spec__1(lean_object*); -static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabRewriteConfig___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___closed__5; @@ -98,10 +100,11 @@ static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__3___closed__1; lean_object* l_Lean_Elab_Tactic_elabTerm(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__6; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withLocation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__4; +static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteLocalDecl(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_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__1; lean_object* lean_nat_div(lean_object*, lean_object*); @@ -113,13 +116,13 @@ lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lea lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getEqnsFor_x3f(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabRewriteConfig___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__2; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteTarget___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__2; @@ -127,7 +130,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Tactic_elabR LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_withRWRulesSeq___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRewriteSeq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteTarget(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -144,20 +147,21 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Tactic_elabR LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteLocalDecl___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_withRWRulesSeq___spec__2___closed__1; static lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___closed__4; -static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4; static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_withRWRulesSeq___spec__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__2; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteTarget___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_withRWRulesSeq___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__7; lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withRWRulesSeq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_withRWRulesSeq___spec__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Tactic_elabRewriteConfig___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__2; +static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteLocalDecl___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteLocalDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -173,7 +177,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabRewrit static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__1; static lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___closed__8; static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_withRWRulesSeq___spec__7___closed__1; -static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__1; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); @@ -182,13 +185,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabRewrit static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq_go___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withRWRulesSeq_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq___closed__2; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabRewriteConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_withRWRulesSeq___spec__7___closed__2; -static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__7; LEAN_EXPORT lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_withRWRulesSeq___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -205,8 +207,8 @@ static lean_object* l_Lean_Elab_Tactic_elabRewriteConfig___closed__9; extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4; +static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3; +static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3; lean_object* l_Lean_Elab_ContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -220,19 +222,19 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Tactic_elabR uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterTR_loop___at_Lean_resolveGlobalConstCore___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq(lean_object*); lean_object* l___private_Lean_Meta_Tactic_Replace_0__Lean_Meta_replaceLocalDeclCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_withRWRulesSeq___closed__3; -static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_withRWRulesSeq___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__4; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_withRWRulesSeq___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__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_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__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_EXPORT lean_object* l_Lean_Elab_Tactic_rewriteTarget___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { @@ -1788,7 +1790,65 @@ return x_63; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_getFVarId(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_11, 0, x_14); +return x_11; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_11); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_15); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_11); +if (x_19 == 0) +{ +return x_11; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_11, 0); +x_21 = lean_ctor_get(x_11, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_11); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; @@ -2170,7 +2230,7 @@ return x_85; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; lean_object* x_15; @@ -2549,7 +2609,7 @@ return x_84; } } } -static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1() { +static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2557,7 +2617,7 @@ x_1 = lean_mk_string_from_bytes("Lean", 4); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2() { +static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2() { _start: { lean_object* x_1; @@ -2565,7 +2625,7 @@ x_1 = lean_mk_string_from_bytes("Parser", 6); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3() { +static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3() { _start: { lean_object* x_1; @@ -2573,7 +2633,7 @@ x_1 = lean_mk_string_from_bytes("Term", 4); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4() { +static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4() { _start: { lean_object* x_1; @@ -2581,19 +2641,19 @@ x_1 = lean_mk_string_from_bytes("explicit", 8); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5() { +static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1; -x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2; -x_3 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3; -x_4 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1; +x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2; +x_3 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3; +x_4 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(lean_object* x_1, uint8_t 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_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4(lean_object* x_1, uint8_t 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) { _start: { uint8_t x_16; @@ -2609,7 +2669,7 @@ lean_ctor_set(x_13, 5, x_18); if (x_2 == 0) { lean_object* x_19; uint8_t x_20; -x_19 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5; +x_19 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5; lean_inc(x_3); x_20 = l_Lean_Syntax_isOfKind(x_3, x_19); if (x_20 == 0) @@ -2638,13 +2698,16 @@ return x_27; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_inc(x_24); +x_28 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1), 10, 1); +lean_closure_set(x_28, 0, x_24); +x_55 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -2653,98 +2716,222 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_24); -x_31 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_30); -if (lean_obj_tag(x_31) == 0) +x_58 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_57); +if (lean_obj_tag(x_58) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_29); +lean_object* x_59; lean_object* x_60; +lean_dec(x_56); +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +x_29 = x_59; +x_30 = x_60; +goto block_54; +} +else +{ +lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_61 = lean_ctor_get(x_58, 1); +lean_inc(x_61); +lean_dec(x_58); +x_62 = 0; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_63 = l_Lean_Elab_Tactic_SavedState_restore(x_56, x_62, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_61); +x_64 = lean_ctor_get(x_63, 1); +lean_inc(x_64); +lean_dec(x_63); +x_65 = lean_box(0); +x_29 = x_65; +x_30 = x_64; +goto block_54; +} +block_54: +{ +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_30); x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); x_33 = lean_ctor_get(x_31, 1); lean_inc(x_33); lean_dec(x_31); -x_34 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_3, x_24, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_33); -return x_34; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_24); +x_34 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_33); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_32); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_4, x_5, x_3, x_24, x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_36); +return x_37; } else { -lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_dec(x_24); -x_35 = lean_ctor_get(x_31, 1); -lean_inc(x_35); -lean_dec(x_31); -x_36 = 0; +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); +lean_dec(x_34); +x_39 = 0; lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_37 = l_Lean_Elab_Tactic_SavedState_restore(x_29, x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_35); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); -x_39 = lean_box(x_5); -x_40 = lean_apply_11(x_4, x_39, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_38); -if (lean_obj_tag(x_40) == 0) +x_40 = l_Lean_Elab_Tactic_SavedState_restore(x_32, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_38); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = lean_box(x_5); +x_43 = lean_apply_11(x_4, x_42, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_41); +if (lean_obj_tag(x_43) == 0) { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +uint8_t x_44; +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -return x_40; +return x_43; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 0); -x_43 = lean_ctor_get(x_40, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_40); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_43, 0); +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_43); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } else { -uint8_t x_45; -x_45 = !lean_is_exclusive(x_40); -if (x_45 == 0) +uint8_t x_48; +x_48 = !lean_is_exclusive(x_43); +if (x_48 == 0) { -return x_40; +return x_43; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_40, 0); -x_47 = lean_ctor_get(x_40, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_40); -x_48 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -return x_48; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_43, 0); +x_50 = lean_ctor_get(x_43, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_43); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } } +else +{ +lean_object* x_52; lean_object* x_53; +lean_dec(x_29); +lean_dec(x_24); +x_52 = lean_box(x_5); +x_53 = lean_apply_11(x_4, x_52, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_30); +return x_53; +} +} +} } } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_dec(x_6); -x_49 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); +lean_inc(x_3); +x_66 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1), 10, 1); +lean_closure_set(x_66, 0, x_3); +x_93 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_96 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_66, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_95); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; lean_object* x_98; +lean_dec(x_94); +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_67 = x_97; +x_68 = x_98; +goto block_92; +} +else +{ +lean_object* x_99; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = 0; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_101 = l_Lean_Elab_Tactic_SavedState_restore(x_94, x_100, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_99); +x_102 = lean_ctor_get(x_101, 1); +lean_inc(x_102); +lean_dec(x_101); +x_103 = lean_box(0); +x_67 = x_103; +x_68 = x_102; +goto block_92; +} +block_92: +{ +if (lean_obj_tag(x_67) == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_69 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -2754,254 +2941,333 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_3); -x_52 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_51); -if (lean_obj_tag(x_52) == 0) +x_72 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_71); +if (lean_obj_tag(x_72) == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_dec(x_50); -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_4, x_5, x_3, x_53, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_54); -return x_55; +lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_dec(x_70); +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); +x_75 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(x_4, x_5, x_3, x_73, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_74); +return x_75; } else { -lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_56 = lean_ctor_get(x_52, 1); -lean_inc(x_56); -lean_dec(x_52); -x_57 = 0; +lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_76 = lean_ctor_get(x_72, 1); +lean_inc(x_76); +lean_dec(x_72); +x_77 = 0; lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_58 = l_Lean_Elab_Tactic_SavedState_restore(x_50, x_57, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_56); -x_59 = lean_ctor_get(x_58, 1); -lean_inc(x_59); -lean_dec(x_58); -x_60 = lean_box(x_5); -x_61 = lean_apply_11(x_4, x_60, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_59); -if (lean_obj_tag(x_61) == 0) +x_78 = l_Lean_Elab_Tactic_SavedState_restore(x_70, x_77, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_76); +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = lean_box(x_5); +x_81 = lean_apply_11(x_4, x_80, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_79); +if (lean_obj_tag(x_81) == 0) { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +uint8_t x_82; +x_82 = !lean_is_exclusive(x_81); +if (x_82 == 0) { -return x_61; +return x_81; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_61); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_81, 0); +x_84 = lean_ctor_get(x_81, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_81); +x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; } } else { -uint8_t x_66; -x_66 = !lean_is_exclusive(x_61); -if (x_66 == 0) +uint8_t x_86; +x_86 = !lean_is_exclusive(x_81); +if (x_86 == 0) { -return x_61; +return x_81; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_61, 0); -x_68 = lean_ctor_get(x_61, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_61); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_81, 0); +x_88 = lean_ctor_get(x_81, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_81); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +return x_89; } } } } +else +{ +lean_object* x_90; lean_object* x_91; +lean_dec(x_67); +x_90 = lean_box(x_5); +x_91 = lean_apply_11(x_4, x_90, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +return x_91; +} +} +} } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_70 = lean_ctor_get(x_13, 0); -x_71 = lean_ctor_get(x_13, 1); -x_72 = lean_ctor_get(x_13, 2); -x_73 = lean_ctor_get(x_13, 3); -x_74 = lean_ctor_get(x_13, 4); -x_75 = lean_ctor_get(x_13, 5); -x_76 = lean_ctor_get(x_13, 6); -x_77 = lean_ctor_get(x_13, 7); -x_78 = lean_ctor_get(x_13, 8); -x_79 = lean_ctor_get(x_13, 9); -x_80 = lean_ctor_get(x_13, 10); -lean_inc(x_80); -lean_inc(x_79); -lean_inc(x_78); -lean_inc(x_77); -lean_inc(x_76); -lean_inc(x_75); -lean_inc(x_74); -lean_inc(x_73); -lean_inc(x_72); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_104 = lean_ctor_get(x_13, 0); +x_105 = lean_ctor_get(x_13, 1); +x_106 = lean_ctor_get(x_13, 2); +x_107 = lean_ctor_get(x_13, 3); +x_108 = lean_ctor_get(x_13, 4); +x_109 = lean_ctor_get(x_13, 5); +x_110 = lean_ctor_get(x_13, 6); +x_111 = lean_ctor_get(x_13, 7); +x_112 = lean_ctor_get(x_13, 8); +x_113 = lean_ctor_get(x_13, 9); +x_114 = lean_ctor_get(x_13, 10); +lean_inc(x_114); +lean_inc(x_113); +lean_inc(x_112); +lean_inc(x_111); +lean_inc(x_110); +lean_inc(x_109); +lean_inc(x_108); +lean_inc(x_107); +lean_inc(x_106); +lean_inc(x_105); +lean_inc(x_104); lean_dec(x_13); -x_81 = l_Lean_replaceRef(x_1, x_75); -lean_dec(x_75); +x_115 = l_Lean_replaceRef(x_1, x_109); +lean_dec(x_109); lean_dec(x_1); -x_82 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_82, 0, x_70); -lean_ctor_set(x_82, 1, x_71); -lean_ctor_set(x_82, 2, x_72); -lean_ctor_set(x_82, 3, x_73); -lean_ctor_set(x_82, 4, x_74); -lean_ctor_set(x_82, 5, x_81); -lean_ctor_set(x_82, 6, x_76); -lean_ctor_set(x_82, 7, x_77); -lean_ctor_set(x_82, 8, x_78); -lean_ctor_set(x_82, 9, x_79); -lean_ctor_set(x_82, 10, x_80); +x_116 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_116, 0, x_104); +lean_ctor_set(x_116, 1, x_105); +lean_ctor_set(x_116, 2, x_106); +lean_ctor_set(x_116, 3, x_107); +lean_ctor_set(x_116, 4, x_108); +lean_ctor_set(x_116, 5, x_115); +lean_ctor_set(x_116, 6, x_110); +lean_ctor_set(x_116, 7, x_111); +lean_ctor_set(x_116, 8, x_112); +lean_ctor_set(x_116, 9, x_113); +lean_ctor_set(x_116, 10, x_114); if (x_2 == 0) { -lean_object* x_83; uint8_t x_84; -x_83 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5; +lean_object* x_117; uint8_t x_118; +x_117 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5; lean_inc(x_3); -x_84 = l_Lean_Syntax_isOfKind(x_3, x_83); -if (x_84 == 0) +x_118 = l_Lean_Syntax_isOfKind(x_3, x_117); +if (x_118 == 0) { -lean_object* x_85; lean_object* x_86; +lean_object* x_119; lean_object* x_120; lean_dec(x_6); -x_85 = lean_box(x_5); -x_86 = lean_apply_11(x_4, x_85, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_15); -return x_86; +x_119 = lean_box(x_5); +x_120 = lean_apply_11(x_4, x_119, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_15); +return x_120; } else { -lean_object* x_87; lean_object* x_88; uint8_t x_89; -x_87 = lean_unsigned_to_nat(1u); -x_88 = l_Lean_Syntax_getArg(x_3, x_87); -lean_inc(x_88); -x_89 = l_Lean_Syntax_isOfKind(x_88, x_6); +lean_object* x_121; lean_object* x_122; uint8_t x_123; +x_121 = lean_unsigned_to_nat(1u); +x_122 = l_Lean_Syntax_getArg(x_3, x_121); +lean_inc(x_122); +x_123 = l_Lean_Syntax_isOfKind(x_122, x_6); lean_dec(x_6); -if (x_89 == 0) +if (x_123 == 0) { -lean_object* x_90; lean_object* x_91; -lean_dec(x_88); -x_90 = lean_box(x_5); -x_91 = lean_apply_11(x_4, x_90, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_15); -return x_91; +lean_object* x_124; lean_object* x_125; +lean_dec(x_122); +x_124 = lean_box(x_5); +x_125 = lean_apply_11(x_4, x_124, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_15); +return x_125; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_92 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_15); -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +lean_inc(x_122); +x_126 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1), 10, 1); +lean_closure_set(x_126, 0, x_122); +x_153 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_15); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +x_155 = lean_ctor_get(x_153, 1); +lean_inc(x_155); +lean_dec(x_153); lean_inc(x_14); -lean_inc(x_82); +lean_inc(x_116); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_88); -x_95 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_88, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_94); -if (lean_obj_tag(x_95) == 0) +x_156 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_126, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_155); +if (lean_obj_tag(x_156) == 0) +{ +lean_object* x_157; lean_object* x_158; +lean_dec(x_154); +x_157 = lean_ctor_get(x_156, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_156, 1); +lean_inc(x_158); +lean_dec(x_156); +x_127 = x_157; +x_128 = x_158; +goto block_152; +} +else +{ +lean_object* x_159; uint8_t x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_159 = lean_ctor_get(x_156, 1); +lean_inc(x_159); +lean_dec(x_156); +x_160 = 0; +lean_inc(x_14); +lean_inc(x_116); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_161 = l_Lean_Elab_Tactic_SavedState_restore(x_154, x_160, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_159); +x_162 = lean_ctor_get(x_161, 1); +lean_inc(x_162); +lean_dec(x_161); +x_163 = lean_box(0); +x_127 = x_163; +x_128 = x_162; +goto block_152; +} +block_152: +{ +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_129 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_128); +x_130 = lean_ctor_get(x_129, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_129, 1); +lean_inc(x_131); +lean_dec(x_129); +lean_inc(x_14); +lean_inc(x_116); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_122); +x_132 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_122, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_131); +if (lean_obj_tag(x_132) == 0) { -lean_object* x_96; lean_object* x_97; lean_object* x_98; -lean_dec(x_93); -x_96 = lean_ctor_get(x_95, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_95, 1); -lean_inc(x_97); -lean_dec(x_95); -x_98 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_3, x_88, x_96, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_97); -return x_98; +lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_dec(x_130); +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_132, 1); +lean_inc(x_134); +lean_dec(x_132); +x_135 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_4, x_5, x_3, x_122, x_133, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_134); +return x_135; } else { -lean_object* x_99; uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -lean_dec(x_88); -x_99 = lean_ctor_get(x_95, 1); -lean_inc(x_99); -lean_dec(x_95); -x_100 = 0; +lean_object* x_136; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +lean_dec(x_122); +x_136 = lean_ctor_get(x_132, 1); +lean_inc(x_136); +lean_dec(x_132); +x_137 = 0; lean_inc(x_14); -lean_inc(x_82); +lean_inc(x_116); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_101 = l_Lean_Elab_Tactic_SavedState_restore(x_93, x_100, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_99); -x_102 = lean_ctor_get(x_101, 1); -lean_inc(x_102); -lean_dec(x_101); -x_103 = lean_box(x_5); -x_104 = lean_apply_11(x_4, x_103, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_102); -if (lean_obj_tag(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_104, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_104, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_107 = x_104; +x_138 = l_Lean_Elab_Tactic_SavedState_restore(x_130, x_137, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_136); +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +lean_dec(x_138); +x_140 = lean_box(x_5); +x_141 = lean_apply_11(x_4, x_140, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_139); +if (lean_obj_tag(x_141) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_144 = x_141; } else { - lean_dec_ref(x_104); - x_107 = lean_box(0); + lean_dec_ref(x_141); + x_144 = lean_box(0); } -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_144)) { + x_145 = lean_alloc_ctor(0, 2, 0); } else { - x_108 = x_107; + x_145 = x_144; } -lean_ctor_set(x_108, 0, x_105); -lean_ctor_set(x_108, 1, x_106); -return x_108; +lean_ctor_set(x_145, 0, x_142); +lean_ctor_set(x_145, 1, x_143); +return x_145; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_109 = lean_ctor_get(x_104, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_104, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_111 = x_104; +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = lean_ctor_get(x_141, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_141, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_148 = x_141; } else { - lean_dec_ref(x_104); - x_111 = lean_box(0); + lean_dec_ref(x_141); + x_148 = lean_box(0); } -if (lean_is_scalar(x_111)) { - x_112 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(1, 2, 0); } else { - x_112 = x_111; + x_149 = x_148; +} +lean_ctor_set(x_149, 0, x_146); +lean_ctor_set(x_149, 1, x_147); +return x_149; +} } -lean_ctor_set(x_112, 0, x_109); -lean_ctor_set(x_112, 1, x_110); -return x_112; +} +else +{ +lean_object* x_150; lean_object* x_151; +lean_dec(x_127); +lean_dec(x_122); +x_150 = lean_box(x_5); +x_151 = lean_apply_11(x_4, x_150, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_128); +return x_151; } } } @@ -3009,16 +3275,74 @@ return x_112; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_dec(x_6); -x_113 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_15); -x_114 = lean_ctor_get(x_113, 0); -lean_inc(x_114); -x_115 = lean_ctor_get(x_113, 1); -lean_inc(x_115); -lean_dec(x_113); +lean_inc(x_3); +x_164 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1), 10, 1); +lean_closure_set(x_164, 0, x_3); +x_191 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_15); +x_192 = lean_ctor_get(x_191, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_191, 1); +lean_inc(x_193); +lean_dec(x_191); lean_inc(x_14); -lean_inc(x_82); +lean_inc(x_116); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_194 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_164, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_193); +if (lean_obj_tag(x_194) == 0) +{ +lean_object* x_195; lean_object* x_196; +lean_dec(x_192); +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_ctor_get(x_194, 1); +lean_inc(x_196); +lean_dec(x_194); +x_165 = x_195; +x_166 = x_196; +goto block_190; +} +else +{ +lean_object* x_197; uint8_t x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_197 = lean_ctor_get(x_194, 1); +lean_inc(x_197); +lean_dec(x_194); +x_198 = 0; +lean_inc(x_14); +lean_inc(x_116); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_199 = l_Lean_Elab_Tactic_SavedState_restore(x_192, x_198, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_197); +x_200 = lean_ctor_get(x_199, 1); +lean_inc(x_200); +lean_dec(x_199); +x_201 = lean_box(0); +x_165 = x_201; +x_166 = x_200; +goto block_190; +} +block_190: +{ +if (lean_obj_tag(x_165) == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; +x_167 = l_Lean_Elab_Tactic_saveState___rarg(x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_166); +x_168 = lean_ctor_get(x_167, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_167, 1); +lean_inc(x_169); +lean_dec(x_167); +lean_inc(x_14); +lean_inc(x_116); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -3026,92 +3350,102 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_3); -x_116 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_115); -if (lean_obj_tag(x_116) == 0) -{ -lean_object* x_117; lean_object* x_118; lean_object* x_119; -lean_dec(x_114); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_116, 1); -lean_inc(x_118); -lean_dec(x_116); -x_119 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_4, x_5, x_3, x_117, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_118); -return x_119; -} -else -{ -lean_object* x_120; uint8_t x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_120 = lean_ctor_get(x_116, 1); -lean_inc(x_120); -lean_dec(x_116); -x_121 = 0; +x_170 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_169); +if (lean_obj_tag(x_170) == 0) +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_dec(x_168); +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_170, 1); +lean_inc(x_172); +lean_dec(x_170); +x_173 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(x_4, x_5, x_3, x_171, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_172); +return x_173; +} +else +{ +lean_object* x_174; uint8_t x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_174 = lean_ctor_get(x_170, 1); +lean_inc(x_174); +lean_dec(x_170); +x_175 = 0; lean_inc(x_14); -lean_inc(x_82); +lean_inc(x_116); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_122 = l_Lean_Elab_Tactic_SavedState_restore(x_114, x_121, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_120); -x_123 = lean_ctor_get(x_122, 1); -lean_inc(x_123); -lean_dec(x_122); -x_124 = lean_box(x_5); -x_125 = lean_apply_11(x_4, x_124, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_82, x_14, x_123); -if (lean_obj_tag(x_125) == 0) -{ -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_126 = lean_ctor_get(x_125, 0); -lean_inc(x_126); -x_127 = lean_ctor_get(x_125, 1); -lean_inc(x_127); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_128 = x_125; +x_176 = l_Lean_Elab_Tactic_SavedState_restore(x_168, x_175, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_174); +x_177 = lean_ctor_get(x_176, 1); +lean_inc(x_177); +lean_dec(x_176); +x_178 = lean_box(x_5); +x_179 = lean_apply_11(x_4, x_178, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_177); +if (lean_obj_tag(x_179) == 0) +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +x_180 = lean_ctor_get(x_179, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_179, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_182 = x_179; } else { - lean_dec_ref(x_125); - x_128 = lean_box(0); + lean_dec_ref(x_179); + x_182 = lean_box(0); } -if (lean_is_scalar(x_128)) { - x_129 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_182)) { + x_183 = lean_alloc_ctor(0, 2, 0); } else { - x_129 = x_128; + x_183 = x_182; } -lean_ctor_set(x_129, 0, x_126); -lean_ctor_set(x_129, 1, x_127); -return x_129; +lean_ctor_set(x_183, 0, x_180); +lean_ctor_set(x_183, 1, x_181); +return x_183; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_130 = lean_ctor_get(x_125, 0); -lean_inc(x_130); -x_131 = lean_ctor_get(x_125, 1); -lean_inc(x_131); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_132 = x_125; +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_184 = lean_ctor_get(x_179, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_179, 1); +lean_inc(x_185); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_186 = x_179; } else { - lean_dec_ref(x_125); - x_132 = lean_box(0); + lean_dec_ref(x_179); + x_186 = lean_box(0); } -if (lean_is_scalar(x_132)) { - x_133 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_186)) { + x_187 = lean_alloc_ctor(1, 2, 0); } else { - x_133 = x_132; + x_187 = x_186; +} +lean_ctor_set(x_187, 0, x_184); +lean_ctor_set(x_187, 1, x_185); +return x_187; } -lean_ctor_set(x_133, 0, x_130); -lean_ctor_set(x_133, 1, x_131); -return x_133; +} +} +else +{ +lean_object* x_188; lean_object* x_189; +lean_dec(x_165); +x_188 = lean_box(x_5); +x_189 = lean_apply_11(x_4, x_188, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_116, x_14, x_166); +return x_189; } } } } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; @@ -3294,14 +3628,14 @@ lean_dec(x_41); x_45 = lean_box(x_36); x_46 = lean_box(x_42); lean_inc(x_1); -x_47 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___boxed), 15, 6); +x_47 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___boxed), 15, 6); lean_closure_set(x_47, 0, x_30); lean_closure_set(x_47, 1, x_45); lean_closure_set(x_47, 2, x_34); lean_closure_set(x_47, 3, x_1); lean_closure_set(x_47, 4, x_46); lean_closure_set(x_47, 5, x_35); -x_48 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4), 11, 1); +x_48 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__5), 11, 1); lean_closure_set(x_48, 0, x_43); lean_inc(x_18); lean_inc(x_17); @@ -3473,7 +3807,7 @@ lean_inc(x_25); x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); lean_dec(x_24); -x_27 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4), 11, 1); +x_27 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__5), 11, 1); lean_closure_set(x_27, 0, x_25); x_28 = l_Lean_Elab_Tactic_withRWRulesSeq___closed__4; lean_inc(x_11); @@ -3663,27 +3997,27 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; x_15 = lean_unbox(x_2); lean_dec(x_2); -x_16 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_1, x_15, 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_16 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_1, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); return x_16; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; lean_object* x_15; x_14 = lean_unbox(x_2); lean_dec(x_2); -x_15 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2(x_1, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(x_1, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); return x_15; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { uint8_t x_16; uint8_t x_17; lean_object* x_18; @@ -3691,7 +4025,7 @@ x_16 = lean_unbox(x_2); lean_dec(x_2); x_17 = lean_unbox(x_5); lean_dec(x_5); -x_18 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3(x_1, x_16, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_18 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4(x_1, x_16, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); return x_18; } } @@ -3735,7 +4069,7 @@ lean_dec(x_2); return x_13; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1() { _start: { lean_object* x_1; @@ -3743,7 +4077,7 @@ x_1 = lean_mk_string_from_bytes("Meta", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2() { _start: { lean_object* x_1; @@ -3751,7 +4085,7 @@ x_1 = lean_mk_string_from_bytes("Rewrite", 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3() { _start: { lean_object* x_1; @@ -3759,33 +4093,33 @@ x_1 = lean_mk_string_from_bytes("Config", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1; -x_2 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1; -x_3 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2; -x_4 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1; +x_2 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1; +x_3 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2; +x_4 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; uint8_t x_10; lean_object* x_11; -x_9 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4; +x_9 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4; x_10 = 0; x_11 = l_Lean_Meta_evalExpr_x27___rarg(x_9, x_1, x_10, x_4, x_5, x_6, x_7, x_8); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679_(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735_(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; @@ -5179,7 +5513,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_elabRewriteConfig___closed__9() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4; +x_2 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -5258,7 +5592,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679_(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_28); +x_29 = l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735_(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_28); lean_dec(x_3); lean_dec(x_2); return x_29; @@ -5708,8 +6042,8 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1; -x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1; +x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2; x_3 = l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__1; x_4 = l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); @@ -5736,7 +6070,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1; x_2 = l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__4; x_3 = l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__1; x_4 = l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__5; @@ -5776,7 +6110,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(64u); +x_1 = lean_unsigned_to_nat(68u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5788,7 +6122,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(71u); +x_1 = lean_unsigned_to_nat(75u); x_2 = lean_unsigned_to_nat(91u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5816,7 +6150,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(64u); +x_1 = lean_unsigned_to_nat(68u); x_2 = lean_unsigned_to_nat(52u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5828,7 +6162,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(64u); +x_1 = lean_unsigned_to_nat(68u); x_2 = lean_unsigned_to_nat(66u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5923,16 +6257,16 @@ l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec_ lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__2); l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__3 = _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__3(); lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1___closed__3); -l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__1); -l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2(); -lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__2); -l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3(); -lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__3); -l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4(); -lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__4); -l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5(); -lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__3___closed__5); +l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__1); +l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__2); +l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3(); +lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__3); +l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4(); +lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__4); +l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5(); +lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__4___closed__5); l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__1 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__1(); lean_mark_persistent(l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__1); l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__2 = _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__2(); @@ -5945,14 +6279,14 @@ l_Lean_Elab_Tactic_withRWRulesSeq___closed__3 = _init_l_Lean_Elab_Tactic_withRWR lean_mark_persistent(l_Lean_Elab_Tactic_withRWRulesSeq___closed__3); l_Lean_Elab_Tactic_withRWRulesSeq___closed__4 = _init_l_Lean_Elab_Tactic_withRWRulesSeq___closed__4(); lean_mark_persistent(l_Lean_Elab_Tactic_withRWRulesSeq___closed__4); -l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__1); -l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__2); -l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__3); -l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1679____closed__4); +l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__1); +l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__2); +l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__3); +l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4 = _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_1735____closed__4); l_Lean_Elab_Tactic_elabRewriteConfig___closed__1 = _init_l_Lean_Elab_Tactic_elabRewriteConfig___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_elabRewriteConfig___closed__1); l_Lean_Elab_Tactic_elabRewriteConfig___closed__2 = _init_l_Lean_Elab_Tactic_elabRewriteConfig___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Simp.c b/stage0/stdlib/Lean/Elab/Tactic/Simp.c index 5fa5e1f0bf70..974ca02ec5df 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Simp.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Simp.c @@ -2044,7 +2044,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_4); @@ -2409,7 +2409,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_3); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Acyclic.c b/stage0/stdlib/Lean/Meta/Tactic/Acyclic.c index 9ecb36e97eed..81b046ec89e5 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Acyclic.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Acyclic.c @@ -394,7 +394,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_4); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c index 8ea67b93a0d8..aa3bc68ea541 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c @@ -13,33 +13,29 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_get_x3f(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Meta_Linear_Cnstr_getBound___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqCnstrKind___boxed(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__outOfBounds___rarg(lean_object*); static lean_object* l_Lean_Meta_Linear_instReprVar___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188_(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_assignment___default; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprCnstr; static lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___closed__2; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_resolve(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_size___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_add_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprAssumptionId; -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3347_(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__9; LEAN_EXPORT lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Linear_getBestBound_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqJustification(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Linear_Poly_eval_x3f___spec__1___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1; static lean_object* l_Lean_Meta_Linear_instInhabitedJustification___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_currVar___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableLtVarInstLTVar___boxed(lean_object*, lean_object*); @@ -49,12 +45,14 @@ static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedState; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_add___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__11; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__12; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_currVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_size___boxed(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2; LEAN_EXPORT lean_object* l_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__1(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); @@ -64,61 +62,58 @@ static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solv LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqPoly___boxed(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); extern uint8_t l_instInhabitedBool; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____boxed(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instInhabitedCnstrKind; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_ordVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_23____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_Linear_CnstrKind_ofNat(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instReprPoly___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Linear_Poly_eval_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instBEqJustification; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22; LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Linear_Cnstr_isUnsat___spec__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqCnstrKind(uint8_t, uint8_t); static lean_object* l_Lean_Meta_Linear_instOrdVar___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491____lambda__1___closed__2; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1; static lean_object* l_Lean_Meta_Linear_Assignment_val___default___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instBEqCnstr; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_getBestBound_x3f(lean_object*, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedJustification; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__15; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15; lean_object* l_Lean_Rat_add(lean_object*, lean_object*); uint8_t l___private_Lean_Data_Rat_0__Lean_beqRat____x40_Lean_Data_Rat___hyg_37_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion___rarg___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431_(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instInhabitedState___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6; static lean_object* l_Lean_Meta_Linear_instBEqCnstrKind___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getNumVars___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_AssumptionId_id___default; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__5; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14; static lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_getMaxVarCoeff(lean_object*); static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__1; size_t lean_usize_of_nat(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__11; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1; -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603_(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__3; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__19; static lean_object* l_Lean_Meta_Linear_Poly_eval_x3f___closed__2; @@ -128,34 +123,37 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Linear_getBest LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_ordVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_23_(lean_object*, lean_object*); lean_object* l_Lean_Rat_inv(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24; static lean_object* l_Lean_Meta_Linear_Poly_getMaxVarCoeff___closed__1; -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593_(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instOrdVar; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3; -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852_(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Poly_add_go___closed__1; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__7; static lean_object* l_Lean_Meta_Linear_instInhabitedCnstr___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_pickAssignment_x3f(lean_object*, uint8_t, lean_object*, uint8_t); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7; uint8_t l_Array_instDecidableEqArray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instReprCnstrKind___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7; LEAN_EXPORT lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3; lean_object* lean_array_to_list(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instReprAssumptionId___closed__1; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__10; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqCnstr___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getBestUpperBound_x3f___boxed(lean_object*); static lean_object* l_Lean_Meta_Linear_instReprJustification___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_scale(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_solve(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Meta_Linear_Cnstr_getBound___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqVar(lean_object*, lean_object*); lean_object* l_Int_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprJustification; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedAssumptionId; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_98____boxed(lean_object*, lean_object*); @@ -165,51 +163,48 @@ static lean_object* l_Lean_Meta_Linear_instBEqJustification___closed__1; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__16; LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqCnstr(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491_(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9; static lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat___closed__4; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__10; LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqPoly(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getBestUpperBound_x3f(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3347____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedAssignment; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_size(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_eval_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprPoly; +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_get___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__8; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__6; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__13; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3503____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_getMaxVarCoeff___boxed(lean_object*); static lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getNumVars(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprCnstrKind; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_shrink___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__18; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__3; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_98_(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7; -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365_(uint8_t, uint8_t); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__12; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491____lambda__1___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__6; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_scale___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__7; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__2; @@ -222,107 +217,112 @@ lean_object* lean_string_length(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqAssumptionId(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instBEqCnstr___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getBestLowerBound_x3f(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__4; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__9; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13; +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_getBound(lean_object*, lean_object*); lean_object* l_instDecidableEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instLTVar; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getBestLowerBound_x3f___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_isStrict___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__8; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5; lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13; static lean_object* l_Lean_Meta_Linear_instReprCnstr___closed__1; uint8_t l_Lean_Rat_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedCnstr; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2; lean_object* l_Std_Format_joinSep___at_Prod_repr___spec__1(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23; lean_object* l_Lean_Rat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_noConfusion___rarg___lambda__1(lean_object*); lean_object* l_Repr_addAppParen(lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_getBestBound_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17; uint8_t lean_int_dec_lt(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqAssumptionId___boxed(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Poly_scale___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Cnstr_isUnsat___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_resolve___closed__1; lean_object* l_Lean_Rat_floor(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_size(lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932_(lean_object*, lean_object*); lean_object* l_Nat_decEq___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_add(lean_object*, lean_object*); lean_object* l_Array_back___rarg(lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Lean_Rat_ceil(lean_object*); static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_resolve___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedPoly; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14; size_t lean_usize_add(size_t, size_t); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Linear_Poly_eval_x3f___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); uint8_t l_Lean_Rat_instDecidableLeRatInstLERat(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_get_x3f___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11; lean_object* lean_int_add(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16; uint8_t lean_int_dec_eq(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11; uint8_t l_Lean_Rat_isInt(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491____boxed(lean_object*, lean_object*); extern lean_object* l_Int_instInhabitedInt; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_eval_x3f___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691____boxed(lean_object*, lean_object*); lean_object* l_Lean_Rat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437_(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18; lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_eval_x3f___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1; +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3503_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_ofNat___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__5; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932____boxed(lean_object*, lean_object*); lean_object* lean_int_neg(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491____closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535____boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* l_Int_decEq___boxed(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_add_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableLtVarInstLTVar(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136_(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10; +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_val___default; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprVar; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_assignCurr(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; static lean_object* l_Prod_repr___at___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____spec__2___closed__6; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqVar___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Poly_eval_x3f___closed__1; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_431____closed__20; -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17; +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521_(uint8_t, uint8_t); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_getMaxVar___boxed(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_toCtorIdx(uint8_t); lean_object* l_Nat_repr(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_491____lambda__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759_(lean_object*, lean_object*); static lean_object* _init_l_Lean_Meta_Linear_instInhabitedVar() { _start: { @@ -2484,7 +2484,7 @@ x_1 = lean_unsigned_to_nat(0u); return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3347_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3503_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -2492,11 +2492,11 @@ x_3 = lean_nat_dec_eq(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3347____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3503____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3347_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3503_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -2522,7 +2522,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; @@ -2559,11 +2559,11 @@ lean_ctor_set_uint8(x_17, sizeof(void*)*1, x_7); return x_17; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -2572,7 +2572,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instReprAssumptionId___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593____boxed), 2, 0); return x_1; } } @@ -2602,7 +2602,7 @@ x_1 = l_Lean_Meta_Linear_instInhabitedJustification___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -2628,7 +2628,7 @@ return x_12; else { uint8_t x_13; -x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(x_4, x_8); +x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(x_4, x_8); if (x_13 == 0) { uint8_t x_14; @@ -2680,11 +2680,11 @@ return x_22; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -2695,7 +2695,7 @@ LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqJustification(lean_object* _start: { uint8_t x_3; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(x_1, x_2); return x_3; } } @@ -2710,7 +2710,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088_(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -2736,7 +2736,7 @@ return x_12; else { uint8_t x_13; -x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932_(x_4, x_8); +x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088_(x_4, x_8); if (x_13 == 0) { uint8_t x_14; @@ -2788,11 +2788,11 @@ return x_22; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -2803,7 +2803,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instBEqJustification___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088____boxed), 2, 0); return x_1; } } @@ -2815,7 +2815,7 @@ x_1 = l_Lean_Meta_Linear_instBEqJustification___closed__1; return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1() { _start: { lean_object* x_1; @@ -2823,21 +2823,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.Justification.combine", 38); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2845,7 +2845,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -2854,7 +2854,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -2863,7 +2863,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6() { _start: { lean_object* x_1; @@ -2871,21 +2871,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.Justification.assumption", 41) return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2893,7 +2893,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -2914,7 +2914,7 @@ x_9 = l_Int_repr(x_3); lean_dec(x_3); x_10 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_10, 0, x_9); -x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3; +x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3; x_12 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_12, 0, x_11); lean_ctor_set(x_12, 1, x_10); @@ -2922,7 +2922,7 @@ x_13 = lean_box(1); x_14 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_14, 0, x_12); lean_ctor_set(x_14, 1, x_13); -x_15 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(x_4, x_7); +x_15 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(x_4, x_7); x_16 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -2939,14 +2939,14 @@ lean_ctor_set(x_20, 1, x_19); x_21 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_13); -x_22 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(x_6, x_7); +x_22 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(x_6, x_7); x_23 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); if (x_8 == 0) { lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; -x_24 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; +x_24 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; x_25 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); @@ -2960,7 +2960,7 @@ return x_28; else { lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; -x_29 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; +x_29 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; x_30 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_23); @@ -2980,15 +2980,15 @@ lean_inc(x_34); lean_dec(x_1); x_35 = lean_unsigned_to_nat(1024u); x_36 = lean_nat_dec_le(x_35, x_2); -x_37 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3437_(x_34, x_35); -x_38 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8; +x_37 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3593_(x_34, x_35); +x_38 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8; x_39 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_39, 0, x_38); lean_ctor_set(x_39, 1, x_37); if (x_36 == 0) { lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; -x_40 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; +x_40 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; x_41 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_39); @@ -3002,7 +3002,7 @@ return x_44; else { lean_object* x_45; lean_object* x_46; uint8_t x_47; lean_object* x_48; lean_object* x_49; -x_45 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; +x_45 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; x_46 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_39); @@ -3016,11 +3016,11 @@ return x_49; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -3029,7 +3029,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instReprJustification___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____boxed), 2, 0); return x_1; } } @@ -3220,7 +3220,7 @@ x_6 = lean_box(x_5); return x_6; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365_(uint8_t x_1, uint8_t x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521_(uint8_t x_1, uint8_t x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -3232,7 +3232,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -3240,7 +3240,7 @@ x_3 = lean_unbox(x_1); lean_dec(x_1); x_4 = lean_unbox(x_2); lean_dec(x_2); -x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365_(x_3, x_4); +x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521_(x_3, x_4); x_6 = lean_box(x_5); return x_6; } @@ -3249,7 +3249,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instBEqCnstrKind___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521____boxed), 2, 0); return x_1; } } @@ -3261,7 +3261,7 @@ x_1 = l_Lean_Meta_Linear_instBEqCnstrKind___closed__1; return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1() { _start: { lean_object* x_1; @@ -3269,33 +3269,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.CnstrKind.eq", 29); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3303,23 +3303,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3327,7 +3327,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7() { _start: { lean_object* x_1; @@ -3335,33 +3335,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.CnstrKind.div", 30); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3369,23 +3369,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3393,7 +3393,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13() { _start: { lean_object* x_1; @@ -3401,33 +3401,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.CnstrKind.lt", 29); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3435,23 +3435,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3459,7 +3459,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19() { _start: { lean_object* x_1; @@ -3467,33 +3467,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Linear.CnstrKind.le", 29); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3501,23 +3501,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -3525,7 +3525,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -3537,14 +3537,14 @@ x_4 = lean_nat_dec_le(x_3, x_2); if (x_4 == 0) { lean_object* x_5; lean_object* x_6; -x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4; +x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4; x_6 = l_Repr_addAppParen(x_5, x_2); return x_6; } else { lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6; +x_7 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -3557,14 +3557,14 @@ x_10 = lean_nat_dec_le(x_9, x_2); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10; +x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10; x_12 = l_Repr_addAppParen(x_11, x_2); return x_12; } else { lean_object* x_13; lean_object* x_14; -x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12; +x_13 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -3577,14 +3577,14 @@ x_16 = lean_nat_dec_le(x_15, x_2); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; -x_17 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16; +x_17 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16; x_18 = l_Repr_addAppParen(x_17, x_2); return x_18; } else { lean_object* x_19; lean_object* x_20; -x_19 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18; +x_19 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -3597,14 +3597,14 @@ x_22 = lean_nat_dec_le(x_21, x_2); if (x_22 == 0) { lean_object* x_23; lean_object* x_24; -x_23 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22; +x_23 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22; x_24 = l_Repr_addAppParen(x_23, x_2); return x_24; } else { lean_object* x_25; lean_object* x_26; -x_25 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24; +x_25 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24; x_26 = l_Repr_addAppParen(x_25, x_2); return x_26; } @@ -3612,13 +3612,13 @@ return x_26; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; x_3 = lean_unbox(x_1); lean_dec(x_1); -x_4 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389_(x_3, x_2); +x_4 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -3627,7 +3627,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instReprCnstrKind___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____boxed), 2, 0); return x_1; } } @@ -3663,7 +3663,7 @@ x_1 = l_Lean_Meta_Linear_instInhabitedCnstr___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -3706,18 +3706,18 @@ return x_17; else { uint8_t x_18; -x_18 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3535_(x_6, x_10); +x_18 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3691_(x_6, x_10); return x_18; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -3728,7 +3728,7 @@ LEAN_EXPORT uint8_t l_Lean_Meta_Linear_instDecidableEqCnstr(lean_object* x_1, le _start: { uint8_t x_3; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4603_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4759_(x_1, x_2); return x_3; } } @@ -3743,7 +3743,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -3755,7 +3755,7 @@ x_7 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); x_8 = lean_ctor_get(x_2, 0); x_9 = lean_ctor_get(x_2, 1); x_10 = lean_ctor_get(x_2, 2); -x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4365_(x_3, x_7); +x_11 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4521_(x_3, x_7); if (x_11 == 0) { uint8_t x_12; @@ -3786,18 +3786,18 @@ return x_17; else { uint8_t x_18; -x_18 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3932_(x_6, x_10); +x_18 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4088_(x_6, x_10); return x_18; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -3808,7 +3808,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instBEqCnstr___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4852____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5008____boxed), 2, 0); return x_1; } } @@ -3820,7 +3820,7 @@ x_1 = l_Lean_Meta_Linear_instBEqCnstr___closed__1; return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1() { _start: { lean_object* x_1; @@ -3828,33 +3828,33 @@ x_1 = lean_mk_string_from_bytes("kind", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2; +x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3; x_2 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_188____closed__5; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3862,7 +3862,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -3871,7 +3871,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6() { _start: { lean_object* x_1; @@ -3879,17 +3879,17 @@ x_1 = lean_mk_string_from_bytes("lhs", 3); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8() { _start: { lean_object* x_1; @@ -3897,17 +3897,17 @@ x_1 = lean_mk_string_from_bytes("rhs", 3); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10() { _start: { lean_object* x_1; @@ -3915,24 +3915,24 @@ x_1 = lean_mk_string_from_bytes("jst", 3); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11() { +static lean_object* _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_4 = lean_unsigned_to_nat(0u); -x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389_(x_3, x_4); -x_6 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5; +x_5 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545_(x_3, x_4); +x_6 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); @@ -3940,7 +3940,7 @@ x_8 = 0; x_9 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_9, 0, x_7); lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_8); -x_10 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4; +x_10 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4; x_11 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); @@ -3952,7 +3952,7 @@ x_14 = lean_box(1); x_15 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); -x_16 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7; +x_16 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7; x_17 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -3979,7 +3979,7 @@ lean_ctor_set(x_26, 1, x_12); x_27 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_14); -x_28 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9; +x_28 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9; x_29 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -4007,7 +4007,7 @@ lean_ctor_set(x_37, 1, x_12); x_38 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_38, 0, x_37); lean_ctor_set(x_38, 1, x_14); -x_39 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11; +x_39 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11; x_40 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_39); @@ -4017,7 +4017,7 @@ lean_ctor_set(x_41, 1, x_18); x_42 = lean_ctor_get(x_1, 2); lean_inc(x_42); lean_dec(x_1); -x_43 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092_(x_42, x_4); +x_43 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248_(x_42, x_4); x_44 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_44, 0, x_22); lean_ctor_set(x_44, 1, x_43); @@ -4045,11 +4045,11 @@ lean_ctor_set_uint8(x_53, sizeof(void*)*1, x_8); return x_53; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -4058,7 +4058,7 @@ static lean_object* _init_l_Lean_Meta_Linear_instReprCnstr___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____boxed), 2, 0); return x_1; } } @@ -4955,7 +4955,7 @@ static lean_object* _init_l_Lean_Meta_Linear_pickAssignment_x3f___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4; x_2 = lean_unsigned_to_nat(1u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4976,7 +4976,7 @@ static lean_object* _init_l_Lean_Meta_Linear_pickAssignment_x3f___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5; +x_1 = l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5; x_2 = lean_unsigned_to_nat(1u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -6174,22 +6174,22 @@ l_Lean_Meta_Linear_instBEqJustification___closed__1 = _init_l_Lean_Meta_Linear_i lean_mark_persistent(l_Lean_Meta_Linear_instBEqJustification___closed__1); l_Lean_Meta_Linear_instBEqJustification = _init_l_Lean_Meta_Linear_instBEqJustification(); lean_mark_persistent(l_Lean_Meta_Linear_instBEqJustification); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__1); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__2); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__3); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__4); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__5); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__6); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__7); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4092____closed__8); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__1); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__2); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__3); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__4); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__5); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__6); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__7); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprJustification____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4248____closed__8); l_Lean_Meta_Linear_instReprJustification___closed__1 = _init_l_Lean_Meta_Linear_instReprJustification___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_instReprJustification___closed__1); l_Lean_Meta_Linear_instReprJustification = _init_l_Lean_Meta_Linear_instReprJustification(); @@ -6201,54 +6201,54 @@ l_Lean_Meta_Linear_instBEqCnstrKind___closed__1 = _init_l_Lean_Meta_Linear_instB lean_mark_persistent(l_Lean_Meta_Linear_instBEqCnstrKind___closed__1); l_Lean_Meta_Linear_instBEqCnstrKind = _init_l_Lean_Meta_Linear_instBEqCnstrKind(); lean_mark_persistent(l_Lean_Meta_Linear_instBEqCnstrKind); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__1); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__2); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__3); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__4); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__5); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__6); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__7); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__8); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__9); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__10); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__11); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__12); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__13); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__14); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__15); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__16); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__17); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__18); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__19); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__20); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__21); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__22); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__23); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4389____closed__24); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__1); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__2); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__3); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__4); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__5); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__6); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__7); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__8); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__9); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__10); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__11); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__12); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__13); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__14); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__15); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__16); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__17); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__18); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__19); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__20); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__21); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__22); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__23); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4545____closed__24); l_Lean_Meta_Linear_instReprCnstrKind___closed__1 = _init_l_Lean_Meta_Linear_instReprCnstrKind___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_instReprCnstrKind___closed__1); l_Lean_Meta_Linear_instReprCnstrKind = _init_l_Lean_Meta_Linear_instReprCnstrKind(); @@ -6261,28 +6261,28 @@ l_Lean_Meta_Linear_instBEqCnstr___closed__1 = _init_l_Lean_Meta_Linear_instBEqCn lean_mark_persistent(l_Lean_Meta_Linear_instBEqCnstr___closed__1); l_Lean_Meta_Linear_instBEqCnstr = _init_l_Lean_Meta_Linear_instBEqCnstr(); lean_mark_persistent(l_Lean_Meta_Linear_instBEqCnstr); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__1); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__2); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__3); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__4); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__5); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__6); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__7); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__8); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__9); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__10); -l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4980____closed__11); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__1); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__2); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__3); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__4); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__5); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__6); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__7); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__8); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__9); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__10); +l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11 = _init_l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_5136____closed__11); l_Lean_Meta_Linear_instReprCnstr___closed__1 = _init_l_Lean_Meta_Linear_instReprCnstr___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_instReprCnstr___closed__1); l_Lean_Meta_Linear_instReprCnstr = _init_l_Lean_Meta_Linear_instReprCnstr(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c index 9bd6ccd3cf00..ed8f2c5425b7 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c @@ -58922,131 +58922,134 @@ return x_23; LEAN_EXPORT lean_object* l_Lean_Meta_dsimpGoal___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_dec(x_7); -x_13 = l_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f___lambda__2___closed__2; -x_14 = lean_unsigned_to_nat(3u); -x_15 = l_Lean_Expr_isAppOfArity(x_4, x_13, x_14); -if (x_15 == 0) +x_13 = l_Lean_Expr_consumeMData(x_4); +x_14 = l_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f___lambda__2___closed__2; +x_15 = lean_unsigned_to_nat(3u); +x_16 = l_Lean_Expr_isAppOfArity(x_13, x_14, x_15); +if (x_16 == 0) { -lean_object* x_16; lean_object* x_17; +lean_object* x_17; lean_object* x_18; +lean_dec(x_13); lean_dec(x_5); -x_16 = lean_box(0); -x_17 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_16, x_8, x_9, x_10, x_11, x_12); -return x_17; +x_17 = lean_box(0); +x_18 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_17, x_8, x_9, x_10, x_11, x_12); +return x_18; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_18 = l_Lean_Expr_appFn_x21(x_4); -x_19 = l_Lean_Expr_appArg_x21(x_18); -lean_dec(x_18); -x_20 = l_Lean_Expr_appArg_x21(x_4); -x_21 = lean_ctor_get(x_8, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_8, 1); +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; uint8_t x_28; +x_19 = l_Lean_Expr_appFn_x21(x_13); +x_20 = l_Lean_Expr_appArg_x21(x_19); +lean_dec(x_19); +x_21 = l_Lean_Expr_appArg_x21(x_13); +lean_dec(x_13); +x_22 = lean_ctor_get(x_8, 0); lean_inc(x_22); -x_23 = lean_ctor_get(x_8, 2); +x_23 = lean_ctor_get(x_8, 1); lean_inc(x_23); -x_24 = lean_ctor_get(x_8, 3); +x_24 = lean_ctor_get(x_8, 2); lean_inc(x_24); -x_25 = lean_ctor_get(x_8, 4); +x_25 = lean_ctor_get(x_8, 3); lean_inc(x_25); -x_26 = lean_ctor_get(x_8, 5); +x_26 = lean_ctor_get(x_8, 4); lean_inc(x_26); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) +x_27 = lean_ctor_get(x_8, 5); +lean_inc(x_27); +x_28 = !lean_is_exclusive(x_22); +if (x_28 == 0) { -uint8_t x_28; lean_object* x_29; lean_object* x_30; -x_28 = 2; -lean_ctor_set_uint8(x_21, 9, x_28); -x_29 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_29, 0, x_21); -lean_ctor_set(x_29, 1, x_22); -lean_ctor_set(x_29, 2, x_23); -lean_ctor_set(x_29, 3, x_24); -lean_ctor_set(x_29, 4, x_25); -lean_ctor_set(x_29, 5, x_26); +uint8_t x_29; lean_object* x_30; lean_object* x_31; +x_29 = 2; +lean_ctor_set_uint8(x_22, 9, x_29); +x_30 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_30, 0, x_22); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_24); +lean_ctor_set(x_30, 3, x_25); +lean_ctor_set(x_30, 4, x_26); +lean_ctor_set(x_30, 5, x_27); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_19); -x_30 = l_Lean_Meta_isExprDefEq(x_19, x_20, x_29, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_20); +x_31 = l_Lean_Meta_isExprDefEq(x_20, x_21, x_30, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_unbox(x_31); -lean_dec(x_31); -if (x_32 == 0) +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_dec(x_19); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_20); lean_dec(x_5); -x_33 = lean_ctor_get(x_30, 1); -lean_inc(x_33); -lean_dec(x_30); -x_34 = lean_box(0); -x_35 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_34, x_8, x_9, x_10, x_11, x_33); -return x_35; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +x_35 = lean_box(0); +x_36 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_35, x_8, x_9, x_10, x_11, x_34); +return x_36; } else { -lean_object* x_36; lean_object* x_37; +lean_object* x_37; lean_object* x_38; lean_dec(x_4); lean_dec(x_1); -x_36 = lean_ctor_get(x_30, 1); -lean_inc(x_36); -lean_dec(x_30); +x_37 = lean_ctor_get(x_31, 1); +lean_inc(x_37); +lean_dec(x_31); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_37 = l_Lean_Meta_mkEqRefl(x_19, x_8, x_9, x_10, x_11, x_36); -if (lean_obj_tag(x_37) == 0) +x_38 = l_Lean_Meta_mkEqRefl(x_20, x_8, x_9, x_10, x_11, x_37); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -lean_dec(x_37); -x_40 = l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(x_6, x_38, x_8, x_9, x_10, x_11, x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(x_6, x_39, x_8, x_9, x_10, x_11, x_40); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_40, 0); -lean_dec(x_42); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_5); -lean_ctor_set(x_43, 1, x_2); -lean_ctor_set(x_40, 0, x_43); -return x_40; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_41, 0); +lean_dec(x_43); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_5); +lean_ctor_set(x_44, 1, x_2); +lean_ctor_set(x_41, 0, x_44); +return x_41; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_40, 1); -lean_inc(x_44); -lean_dec(x_40); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_5); -lean_ctor_set(x_45, 1, x_2); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_41, 1); +lean_inc(x_45); +lean_dec(x_41); x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_ctor_set(x_46, 0, x_5); +lean_ctor_set(x_46, 1, x_2); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +return x_47; } } else { -uint8_t x_47; +uint8_t x_48; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -59054,31 +59057,31 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_47 = !lean_is_exclusive(x_37); -if (x_47 == 0) +x_48 = !lean_is_exclusive(x_38); +if (x_48 == 0) { -return x_37; +return x_38; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_37, 0); -x_49 = lean_ctor_get(x_37, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_38, 0); +x_50 = lean_ctor_get(x_38, 1); +lean_inc(x_50); lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_37); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_dec(x_38); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } } else { -uint8_t x_51; -lean_dec(x_19); +uint8_t x_52; +lean_dec(x_20); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -59088,137 +59091,137 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_51 = !lean_is_exclusive(x_30); -if (x_51 == 0) +x_52 = !lean_is_exclusive(x_31); +if (x_52 == 0) { -return x_30; +return x_31; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_30, 0); -x_53 = lean_ctor_get(x_30, 1); +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_31, 0); +x_54 = lean_ctor_get(x_31, 1); +lean_inc(x_54); lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_30); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_dec(x_31); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } else { -uint8_t x_55; uint8_t x_56; uint8_t x_57; uint8_t x_58; uint8_t x_59; uint8_t x_60; uint8_t x_61; uint8_t x_62; uint8_t x_63; uint8_t x_64; uint8_t x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_55 = lean_ctor_get_uint8(x_21, 0); -x_56 = lean_ctor_get_uint8(x_21, 1); -x_57 = lean_ctor_get_uint8(x_21, 2); -x_58 = lean_ctor_get_uint8(x_21, 3); -x_59 = lean_ctor_get_uint8(x_21, 4); -x_60 = lean_ctor_get_uint8(x_21, 5); -x_61 = lean_ctor_get_uint8(x_21, 6); -x_62 = lean_ctor_get_uint8(x_21, 7); -x_63 = lean_ctor_get_uint8(x_21, 8); -x_64 = lean_ctor_get_uint8(x_21, 10); -x_65 = lean_ctor_get_uint8(x_21, 11); -lean_dec(x_21); -x_66 = 2; -x_67 = lean_alloc_ctor(0, 0, 12); -lean_ctor_set_uint8(x_67, 0, x_55); -lean_ctor_set_uint8(x_67, 1, x_56); -lean_ctor_set_uint8(x_67, 2, x_57); -lean_ctor_set_uint8(x_67, 3, x_58); -lean_ctor_set_uint8(x_67, 4, x_59); -lean_ctor_set_uint8(x_67, 5, x_60); -lean_ctor_set_uint8(x_67, 6, x_61); -lean_ctor_set_uint8(x_67, 7, x_62); -lean_ctor_set_uint8(x_67, 8, x_63); -lean_ctor_set_uint8(x_67, 9, x_66); -lean_ctor_set_uint8(x_67, 10, x_64); -lean_ctor_set_uint8(x_67, 11, x_65); -x_68 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_22); -lean_ctor_set(x_68, 2, x_23); -lean_ctor_set(x_68, 3, x_24); -lean_ctor_set(x_68, 4, x_25); -lean_ctor_set(x_68, 5, x_26); +uint8_t x_56; uint8_t x_57; uint8_t x_58; uint8_t x_59; uint8_t x_60; uint8_t x_61; uint8_t x_62; uint8_t x_63; uint8_t x_64; uint8_t x_65; uint8_t x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_56 = lean_ctor_get_uint8(x_22, 0); +x_57 = lean_ctor_get_uint8(x_22, 1); +x_58 = lean_ctor_get_uint8(x_22, 2); +x_59 = lean_ctor_get_uint8(x_22, 3); +x_60 = lean_ctor_get_uint8(x_22, 4); +x_61 = lean_ctor_get_uint8(x_22, 5); +x_62 = lean_ctor_get_uint8(x_22, 6); +x_63 = lean_ctor_get_uint8(x_22, 7); +x_64 = lean_ctor_get_uint8(x_22, 8); +x_65 = lean_ctor_get_uint8(x_22, 10); +x_66 = lean_ctor_get_uint8(x_22, 11); +lean_dec(x_22); +x_67 = 2; +x_68 = lean_alloc_ctor(0, 0, 12); +lean_ctor_set_uint8(x_68, 0, x_56); +lean_ctor_set_uint8(x_68, 1, x_57); +lean_ctor_set_uint8(x_68, 2, x_58); +lean_ctor_set_uint8(x_68, 3, x_59); +lean_ctor_set_uint8(x_68, 4, x_60); +lean_ctor_set_uint8(x_68, 5, x_61); +lean_ctor_set_uint8(x_68, 6, x_62); +lean_ctor_set_uint8(x_68, 7, x_63); +lean_ctor_set_uint8(x_68, 8, x_64); +lean_ctor_set_uint8(x_68, 9, x_67); +lean_ctor_set_uint8(x_68, 10, x_65); +lean_ctor_set_uint8(x_68, 11, x_66); +x_69 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_23); +lean_ctor_set(x_69, 2, x_24); +lean_ctor_set(x_69, 3, x_25); +lean_ctor_set(x_69, 4, x_26); +lean_ctor_set(x_69, 5, x_27); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_19); -x_69 = l_Lean_Meta_isExprDefEq(x_19, x_20, x_68, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_69) == 0) +lean_inc(x_20); +x_70 = l_Lean_Meta_isExprDefEq(x_20, x_21, x_69, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_70; uint8_t x_71; -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_unbox(x_70); -lean_dec(x_70); -if (x_71 == 0) +lean_object* x_71; uint8_t x_72; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_unbox(x_71); +lean_dec(x_71); +if (x_72 == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -lean_dec(x_19); +lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_dec(x_20); lean_dec(x_5); -x_72 = lean_ctor_get(x_69, 1); -lean_inc(x_72); -lean_dec(x_69); -x_73 = lean_box(0); -x_74 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_73, x_8, x_9, x_10, x_11, x_72); -return x_74; +x_73 = lean_ctor_get(x_70, 1); +lean_inc(x_73); +lean_dec(x_70); +x_74 = lean_box(0); +x_75 = l_Lean_Meta_dsimpGoal___lambda__4(x_1, x_2, x_3, x_4, x_6, x_74, x_8, x_9, x_10, x_11, x_73); +return x_75; } else { -lean_object* x_75; lean_object* x_76; +lean_object* x_76; lean_object* x_77; lean_dec(x_4); lean_dec(x_1); -x_75 = lean_ctor_get(x_69, 1); -lean_inc(x_75); -lean_dec(x_69); +x_76 = lean_ctor_get(x_70, 1); +lean_inc(x_76); +lean_dec(x_70); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_76 = l_Lean_Meta_mkEqRefl(x_19, x_8, x_9, x_10, x_11, x_75); -if (lean_obj_tag(x_76) == 0) +x_77 = l_Lean_Meta_mkEqRefl(x_20, x_8, x_9, x_10, x_11, x_76); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(x_6, x_77, x_8, x_9, x_10, x_11, x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(x_6, x_78, x_8, x_9, x_10, x_11, x_79); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -x_80 = lean_ctor_get(x_79, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_81 = x_79; +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_82 = x_80; } else { - lean_dec_ref(x_79); - x_81 = lean_box(0); + lean_dec_ref(x_80); + x_82 = lean_box(0); } -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_5); -lean_ctor_set(x_82, 1, x_2); -if (lean_is_scalar(x_81)) { - x_83 = lean_alloc_ctor(0, 2, 0); +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_5); +lean_ctor_set(x_83, 1, x_2); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); } else { - x_83 = x_81; + x_84 = x_82; } -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_80); -return x_83; +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -59226,33 +59229,33 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_84 = lean_ctor_get(x_76, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_76, 1); +x_85 = lean_ctor_get(x_77, 0); lean_inc(x_85); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_86 = x_76; +x_86 = lean_ctor_get(x_77, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_87 = x_77; } else { - lean_dec_ref(x_76); - x_86 = lean_box(0); + lean_dec_ref(x_77); + x_87 = lean_box(0); } -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(1, 2, 0); } else { - x_87 = x_86; + x_88 = x_87; } -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; +lean_ctor_set(x_88, 0, x_85); +lean_ctor_set(x_88, 1, x_86); +return x_88; } } } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_19); +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_20); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -59262,26 +59265,26 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_88 = lean_ctor_get(x_69, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_69, 1); +x_89 = lean_ctor_get(x_70, 0); lean_inc(x_89); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_90 = x_69; +x_90 = lean_ctor_get(x_70, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_91 = x_70; } else { - lean_dec_ref(x_69); - x_90 = lean_box(0); + lean_dec_ref(x_70); + x_91 = lean_box(0); } -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_91)) { + x_92 = lean_alloc_ctor(1, 2, 0); } else { - x_91 = x_90; + x_92 = x_91; } -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_89); -return x_91; +lean_ctor_set(x_92, 0, x_89); +lean_ctor_set(x_92, 1, x_90); +return x_92; } } } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/Types.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/Types.c index bfc6523d9d78..86058fc4b72e 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/Types.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/Types.c @@ -206,7 +206,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 5, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 6, x_5); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 7, x_4); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 8, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 9, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 10, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 11, x_3); lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 12, x_4); diff --git a/tests/lean/allFieldForConstants.lean b/tests/lean/allFieldForConstants.lean index b89e333f4193..d0605b565e9a 100644 --- a/tests/lean/allFieldForConstants.lean +++ b/tests/lean/allFieldForConstants.lean @@ -105,7 +105,7 @@ mutual theorem listStringLen_flatList (cs : List Foo) : listStringLen (flatList cs) = textLengthList cs := by match cs with - | [] => simp + | [] => simp [listStringLen] | f :: fs => simp [listStringLen_append, listStringLen_flatList fs, listStringLen_flat f] end diff --git a/tests/lean/letFun.lean b/tests/lean/letFun.lean index 15aa19971042..796f572f3121 100644 --- a/tests/lean/letFun.lean +++ b/tests/lean/letFun.lean @@ -7,4 +7,4 @@ example (a b : Nat) (h1 : a = 0) (h2 : b = 0) : (let_fun x := a + 1; x + x) > b := by simp (config := { beta := false }) [h1] trace_state - simp [h2] + simp (config := { decide := true }) [h2] diff --git a/tests/lean/matchOfNatIssue.lean b/tests/lean/matchOfNatIssue.lean index 0ffdce3d4fcb..7619026464ec 100644 --- a/tests/lean/matchOfNatIssue.lean +++ b/tests/lean/matchOfNatIssue.lean @@ -1,7 +1,7 @@ example (x : Int) (h : x = 2) : Int.div 2 1 = x := by simp [Int.div] trace_state - simp [h] + simp (config := { decide := true }) [h] example (n : Nat) : Int.div (Int.ofNat n) (Int.ofNat 0) = Int.ofNat (n / 0) := by simp [Int.div] diff --git a/tests/lean/run/1293.lean b/tests/lean/run/1293.lean index ee798f741340..6834e8df7019 100644 --- a/tests/lean/run/1293.lean +++ b/tests/lean/run/1293.lean @@ -15,7 +15,7 @@ instance {arr : Array String} {f : String → String} {n : Nat} : Coe (Array (Id def store1 : Store := { arr := #["a", "b", "c", "d", "e"] - ids := #[⟨2, by simp⟩] + ids := #[⟨2, by decide⟩] } def tryCoeStore := { diff --git a/tests/lean/run/1302.lean b/tests/lean/run/1302.lean index 0861b351d76f..0cc9fa7d6527 100644 --- a/tests/lean/run/1302.lean +++ b/tests/lean/run/1302.lean @@ -1,6 +1,6 @@ @[simp] theorem get_cons_zero {as : List α} : (a :: as).get ⟨0, Nat.zero_lt_succ _⟩ = a := rfl -example (a b c : α) : [a, b, c].get ⟨0, by simp⟩ = a := by +example (a b c : α) : [a, b, c].get ⟨0, by simp (config := { decide := true })⟩ = a := by simp example (a : Bool) : (a :: as).get ⟨0, by simp_arith⟩ = a := by @@ -9,5 +9,5 @@ example (a : Bool) : (a :: as).get ⟨0, by simp_arith⟩ = a := by example (a : Bool) : (a :: as).get ⟨0, by simp_arith⟩ = a := by simp -example (a b c : α) : [a, b, c].get ⟨0, by simp⟩ = a := by +example (a b c : α) : [a, b, c].get ⟨0, by simp (config := { decide := true })⟩ = a := by rw [get_cons_zero] diff --git a/tests/lean/run/1380.lean b/tests/lean/run/1380.lean index d5816d8a6c3e..248837b8551a 100644 --- a/tests/lean/run/1380.lean +++ b/tests/lean/run/1380.lean @@ -4,6 +4,6 @@ theorem Nat.lt_succ_iff {m n : Nat} : m < succ n ↔ m ≤ n := sorry variable (n v₁ v₂) (hv₁: v₁ < n + 1) (hv₂: v₂ < n + 1) theorem foo (_: ¬ Fin.mk v₂ hv₂ = Fin.mk v₁ hv₁ ): True := trivial set_option trace.Meta.Tactic.simp true in -example (hv: v₁ < v₂) : True := foo n v₁ v₂ ‹_› ‹_› (by simp only[hv, Fin.mk.injEq, Nat.ne_of_gt, Nat.lt_succ_iff]) +example (hv: v₁ < v₂) : True := foo n v₁ v₂ ‹_› ‹_› (by simp (config := { decide := true }) only [hv, Fin.mk.injEq, Nat.ne_of_gt, Nat.lt_succ_iff]) #check Fin.mk.injEq diff --git a/tests/lean/run/1921.lean b/tests/lean/run/1921.lean index 80e8f4d4096a..bdde9e9c3d29 100644 --- a/tests/lean/run/1921.lean +++ b/tests/lean/run/1921.lean @@ -1,9 +1,9 @@ @[simp] theorem Array.size_singleton : #[a].size = 1 := rfl -@[simp] theorem USize.not_size_le_one : ¬ USize.size ≤ 1 := by cases usize_size_eq <;> simp [*] +@[simp] theorem USize.not_size_le_one : ¬ USize.size ≤ 1 := by cases usize_size_eq <;> simp (config := { decide := true }) [*] def f := #[true].any id 0 USize.size -- `native_decide` used to prove `false` here, due to a bug in `Array.anyMUnsafe`. example : f = true := by native_decide -example : f = true := by simp [f, Array.any, Array.anyM] +example : f = true := by simp (config := { decide := true }) [f, Array.any, Array.anyM] diff --git a/tests/lean/run/891.lean b/tests/lean/run/891.lean index 26d300871334..81bc91ca4538 100644 --- a/tests/lean/run/891.lean +++ b/tests/lean/run/891.lean @@ -44,7 +44,7 @@ example : f 'b' n = 2 := by simp[f] example : f 'c' n = 3 := by - simp[f] + simp (config := { decide := true }) [f] def g : String → Nat → Nat | "hello", _ => 1 @@ -58,7 +58,7 @@ example : g "world" n = 2 := by simp[g] example : g "abc" n = 3 := by - simp[g] + simp (config := { decide := true }) [g] def fn : Fin 8 → Nat → Nat | 2, _ => 1 diff --git a/tests/lean/run/def10.lean b/tests/lean/run/def10.lean index 874119b304ae..e1335b9c6071 100644 --- a/tests/lean/run/def10.lean +++ b/tests/lean/run/def10.lean @@ -27,4 +27,4 @@ theorem ex6 : g x y z > 0 := by split next => decide next => decide - next a b c h₁ h₂ => simp [f_eq h₁] + next a b c h₁ h₂ => simp (config := { decide := true }) [f_eq h₁] diff --git a/tests/lean/run/defaultEliminator.lean b/tests/lean/run/defaultEliminator.lean index fa67666a9188..bcd279164f06 100644 --- a/tests/lean/run/defaultEliminator.lean +++ b/tests/lean/run/defaultEliminator.lean @@ -28,4 +28,4 @@ example (x y : Nat) : f x y > 0 := by | succ_succ x y ih => simp [f, ih] example (x y : Nat) : f x y > 0 := by - induction x, y <;> simp [f, *] + induction x, y <;> simp (config := { decide := true }) [f, *] diff --git a/tests/lean/run/eqnsAtSimp.lean b/tests/lean/run/eqnsAtSimp.lean index ba691658cd72..a296c5f0f778 100644 --- a/tests/lean/run/eqnsAtSimp.lean +++ b/tests/lean/run/eqnsAtSimp.lean @@ -15,5 +15,5 @@ decreasing_by theorem isEven_double (x : Nat) : isEven (2 * x) = true := by induction x with - | zero => simp + | zero => simp [isEven] | succ x ih => simp [Nat.mul_succ, Nat.add_succ, isEven, isOdd, ih] diff --git a/tests/lean/run/maze.lean b/tests/lean/run/maze.lean index a55d9eb6e0bf..431aaecdc5d2 100644 --- a/tests/lean/run/maze.lean +++ b/tests/lean/run/maze.lean @@ -292,5 +292,5 @@ def maze1 := ┌───┐ def foo : can_escape maze1 := by apply step_west set_option trace.Meta.debug true in - simp + simp (config := { decide := true }) out diff --git a/tests/lean/run/mergeSortCPDT.lean b/tests/lean/run/mergeSortCPDT.lean index d7a7ccca4a91..92bf11914dc6 100644 --- a/tests/lean/run/mergeSortCPDT.lean +++ b/tests/lean/run/mergeSortCPDT.lean @@ -26,8 +26,8 @@ theorem List.length_split_of_atLeast2 {as : List α} (h : as.atLeast2) : as.spli match as with | [] => simp at h | [_] => simp at h - | [_, _] => simp [split] - | [_, _, _] => simp [split] + | [_, _] => simp (config := { decide := true }) [split] + | [_, _, _] => simp (config := { decide := true }) [split] | a::b::c::d::as => -- TODO: simplify using linear arith and more automation have : (c::d::as).atLeast2 := by simp_arith diff --git a/tests/lean/run/mutualDefThms.lean b/tests/lean/run/mutualDefThms.lean index 5b62402c1136..a20fee4ffcc4 100644 --- a/tests/lean/run/mutualDefThms.lean +++ b/tests/lean/run/mutualDefThms.lean @@ -54,7 +54,7 @@ mutual theorem listStringLen_flatList (cs : List Foo) : listStringLen (flatList cs) = textLengthList cs := by match cs with - | [] => simp + | [] => simp [listStringLen] | f :: fs => simp [listStringLen_append, listStringLen_flatList fs, listStringLen_flat f] end diff --git a/tests/lean/run/set.lean b/tests/lean/run/set.lean index 82c24a9b0c1c..c1238693617a 100644 --- a/tests/lean/run/set.lean +++ b/tests/lean/run/set.lean @@ -8,7 +8,7 @@ def Set.pred (p : α → Prop) : Set α := p notation "{" a "|" p "}" => Set.pred (fun a => p) theorem ex1 : (1, 3) ∈ { (n, m) | n < 2 ∧ m < 5 } := by - simp [Set.in, Set.pred] + simp (config := { decide := true }) [Set.in, Set.pred] def Set.union (s₁ s₂ : Set α) : Set α := { a | a ∈ s₁ ∨ a ∈ s₂ } diff --git a/tests/lean/run/simp6.lean b/tests/lean/run/simp6.lean index 64f36a558c05..c9006bab7695 100644 --- a/tests/lean/run/simp6.lean +++ b/tests/lean/run/simp6.lean @@ -16,13 +16,13 @@ theorem ex5 : (10 = 20) = False := #print ex5 theorem ex6 : (if "hello" = "world" then 1 else 2) = 2 := - by simp + by simp (config := { decide := true }) #print ex6 theorem ex7 : (if "hello" = "world" then 1 else 2) = 2 := by fail_if_success simp (config := { decide := false }) - simp + simp (config := { decide := true }) theorem ex8 : (10 + 2000 = 20) = False := by simp @@ -32,4 +32,4 @@ def fact : Nat → Nat | x+1 => (x+1) * fact x theorem ex9 : (if fact 100 > 10 then true else false) = true := - by simp + by simp (config := { decide := true }) diff --git a/tests/lean/run/simpDecide.lean b/tests/lean/run/simpDecide.lean new file mode 100644 index 000000000000..cc7464372b7b --- /dev/null +++ b/tests/lean/run/simpDecide.lean @@ -0,0 +1,18 @@ +example : 0 < 4 := by decide + +example : 0 < 4 := by + fail_if_success { simp only } + simp (config := { decide := true }) only + +def fib : Nat → Nat +| 0 => 0 +| 1 => 1 +| n+2 => fib (n+1) + fib n + +theorem fib_two : fib 2 = 1 := rfl + +example : 1 = fib (1 + 1) := by + fail_if_success { simp only [fib_two] } + simp (config := { decide := true }) only [fib_two] + +example : 1 = fib (1 + 1) := by simp only [fib_two, (by decide : 1 + 1 = 2)] diff --git a/tests/lean/run/simp_all.lean b/tests/lean/run/simp_all.lean index 60054b2fda9a..c9dac3d7e2b9 100644 --- a/tests/lean/run/simp_all.lean +++ b/tests/lean/run/simp_all.lean @@ -13,7 +13,7 @@ theorem ex3 (h₁ : a = 0) (h₂ : a + b = 0) : f (b + c) = c := by simp [h₂] theorem ex4 (h₁ : a = f a) (h₂ : b + 0 = 0) : f b = 0 := by - simp_all [-h₁] + simp_all (config := { decide := true }) [-h₁] theorem ex5 (h₁ : a = f a) (h₂ : b + 0 = 0) : f (b + a) = a := by simp_all [-h₁, f] diff --git a/tests/lean/unfold1.lean b/tests/lean/unfold1.lean index 702ee1ee886d..6a77120289f3 100644 --- a/tests/lean/unfold1.lean +++ b/tests/lean/unfold1.lean @@ -11,7 +11,7 @@ decreasing_by apply Nat.lt_succ_self theorem isEven_double (x : Nat) : isEven (2 * x) = true := by induction x with - | zero => simp + | zero => simp [isEven] | succ x ih => unfold isEven trace_state